From af93e4cf8b1a839d21499b3b9737bb8904edcae8 Mon Sep 17 00:00:00 2001 From: letouzey Date: Thu, 29 Apr 2010 13:50:31 +0000 Subject: Remove the svn-specific $Id$ annotations - Many of them were broken, some of them after Pierre B's rework of mli for ocamldoc, but not only (many bad annotation, many files with no svn property about Id, etc) - Useless for those of us that work with git-svn (and a fortiori in a forthcoming git-only setting) - Even in svn, they seem to be of little interest git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12972 85f007b7-540e-0410-9357-904b9bb8a0f7 --- Makefile | 2 -- Makefile.build | 2 -- checker/check.ml | 2 -- checker/checker.ml | 2 -- checker/closure.ml | 2 -- checker/closure.mli | 2 -- checker/indtypes.ml | 2 -- checker/indtypes.mli | 2 -- checker/inductive.ml | 2 -- checker/inductive.mli | 2 -- checker/modops.ml | 2 -- checker/modops.mli | 2 -- checker/reduction.ml | 2 -- checker/reduction.mli | 2 -- checker/safe_typing.ml | 2 -- checker/safe_typing.mli | 2 -- checker/subtyping.ml | 2 -- checker/subtyping.mli | 2 -- checker/term.ml | 2 -- checker/type_errors.ml | 2 -- checker/type_errors.mli | 2 -- checker/typeops.ml | 2 -- checker/typeops.mli | 2 -- checker/validate.ml | 2 -- config/coq_config.mli | 2 -- configure | 1 - doc/common/macros.tex | 2 -- doc/common/title.tex | 1 - doc/refman/Extraction.tex | 2 -- doc/refman/RefMan-add.tex | 2 -- doc/refman/RefMan-cic.tex | 2 -- doc/refman/RefMan-coi.tex | 1 - doc/refman/RefMan-com.tex | 2 -- doc/refman/RefMan-gal.tex | 1 - doc/refman/RefMan-ide.tex | 2 -- doc/refman/RefMan-ind.tex | 1 - doc/refman/RefMan-int.tex | 2 -- doc/refman/RefMan-lib.tex | 2 -- doc/refman/RefMan-modr.tex | 2 -- doc/refman/RefMan-oth.tex | 2 -- doc/refman/RefMan-pre.tex | 2 -- doc/refman/RefMan-pro.tex | 2 -- doc/refman/RefMan-syn.tex | 2 -- doc/refman/RefMan-tac.tex | 2 -- doc/refman/RefMan-uti.tex | 2 -- doc/refman/Reference-Manual.tex | 1 - doc/stdlib/Library.tex | 1 - doc/tutorial/Tutorial.tex | 1 - ide/command_windows.ml | 2 -- ide/command_windows.mli | 2 -- ide/config_lexer.mll | 2 -- ide/config_parser.mly | 2 -- ide/coq.ml | 2 -- ide/coq.mli | 2 -- ide/coq_commands.ml | 2 -- ide/coq_lex.mll | 2 -- ide/coq_tactics.ml | 2 -- ide/coq_tactics.mli | 2 -- ide/coqide.ml | 2 -- ide/coqide.mli | 2 -- ide/gtk_parsing.ml | 2 -- ide/highlight.mll | 2 -- ide/ideproof.ml | 2 -- ide/ideutils.ml | 2 -- ide/ideutils.mli | 2 -- ide/preferences.ml | 2 -- ide/preferences.mli | 2 -- ide/tags.ml | 2 -- ide/typed_notebook.ml | 2 -- ide/undo.ml | 2 -- ide/undo_lablgtk_ge212.mli | 2 -- ide/undo_lablgtk_ge26.mli | 2 -- ide/undo_lablgtk_lt26.mli | 2 -- ide/utf8_convert.mll | 2 -- ide/utils/config_file.ml | 2 -- interp/constrextern.ml | 2 -- interp/constrextern.mli | 2 -- interp/constrintern.ml | 2 -- interp/constrintern.mli | 2 -- interp/coqlib.ml | 2 -- interp/coqlib.mli | 2 -- interp/dumpglob.ml | 2 -- interp/dumpglob.mli | 3 --- interp/genarg.ml | 2 -- interp/genarg.mli | 2 -- interp/implicit_quantifiers.ml | 2 -- interp/implicit_quantifiers.mli | 2 -- interp/modintern.ml | 2 -- interp/modintern.mli | 2 -- interp/notation.ml | 2 -- interp/notation.mli | 2 -- interp/ppextend.ml | 2 -- interp/ppextend.mli | 2 -- interp/reserve.ml | 2 -- interp/reserve.mli | 2 -- interp/smartlocate.ml | 2 -- interp/smartlocate.mli | 2 -- interp/syntax_def.ml | 2 -- interp/syntax_def.mli | 2 -- interp/topconstr.ml | 2 -- interp/topconstr.mli | 2 -- kernel/byterun/int64_emul.h | 2 -- kernel/byterun/int64_native.h | 2 -- kernel/closure.ml | 2 -- kernel/closure.mli | 2 -- kernel/conv_oracle.ml | 2 -- kernel/conv_oracle.mli | 2 -- kernel/cooking.ml | 2 -- kernel/cooking.mli | 2 -- kernel/declarations.ml | 2 -- kernel/declarations.mli | 2 -- kernel/entries.ml | 2 -- kernel/entries.mli | 2 -- kernel/environ.ml | 2 -- kernel/environ.mli | 2 -- kernel/esubst.ml | 2 -- kernel/esubst.mli | 2 -- kernel/indtypes.ml | 2 -- kernel/indtypes.mli | 2 -- kernel/inductive.ml | 2 -- kernel/inductive.mli | 2 -- kernel/mod_subst.ml | 2 -- kernel/mod_subst.mli | 2 -- kernel/mod_typing.ml | 2 -- kernel/mod_typing.mli | 2 -- kernel/modops.ml | 2 -- kernel/modops.mli | 2 -- kernel/names.ml | 2 -- kernel/names.mli | 2 -- kernel/pre_env.ml | 2 -- kernel/pre_env.mli | 2 -- kernel/reduction.ml | 2 -- kernel/reduction.mli | 2 -- kernel/retroknowledge.ml | 2 -- kernel/retroknowledge.mli | 2 -- kernel/safe_typing.ml | 2 -- kernel/safe_typing.mli | 2 -- kernel/sign.ml | 2 -- kernel/sign.mli | 2 -- kernel/subtyping.ml | 2 -- kernel/subtyping.mli | 2 -- kernel/term.ml | 2 -- kernel/term.mli | 2 -- kernel/term_typing.ml | 2 -- kernel/term_typing.mli | 2 -- kernel/type_errors.ml | 2 -- kernel/type_errors.mli | 2 -- kernel/typeops.ml | 2 -- kernel/typeops.mli | 2 -- kernel/univ.ml | 2 -- kernel/univ.mli | 2 -- kernel/vm.ml | 2 -- lib/bigint.ml | 2 -- lib/bigint.mli | 2 -- lib/dnet.ml | 2 -- lib/dnet.mli | 2 -- lib/dyn.ml | 2 -- lib/dyn.mli | 2 -- lib/explore.ml | 2 -- lib/explore.mli | 2 -- lib/flags.ml | 2 -- lib/flags.mli | 2 -- lib/gmap.ml | 1 - lib/gmap.mli | 2 -- lib/gmapl.ml | 2 -- lib/gmapl.mli | 2 -- lib/gset.ml | 2 -- lib/gset.mli | 2 -- lib/hashcons.ml | 2 -- lib/hashcons.mli | 2 -- lib/heap.ml | 2 -- lib/heap.mli | 2 -- lib/option.ml | 2 -- lib/option.mli | 2 -- lib/pp.ml4 | 2 -- lib/pp.mli | 2 -- lib/pp_control.ml | 2 -- lib/pp_control.mli | 2 -- lib/predicate.ml | 2 -- lib/predicate.mli | 2 -- lib/profile.ml | 2 -- lib/profile.mli | 2 -- lib/rtree.ml | 2 -- lib/rtree.mli | 2 -- lib/safe_marshal.ml | 2 -- lib/store.ml | 2 -- lib/store.mli | 2 -- lib/system.ml | 2 -- lib/system.mli | 2 -- lib/tlm.ml | 2 -- lib/tlm.mli | 2 -- lib/util.ml | 2 -- lib/util.mli | 2 -- library/decl_kinds.ml | 2 -- library/decl_kinds.mli | 2 -- library/declare.ml | 2 -- library/declare.mli | 2 -- library/declaremods.ml | 2 -- library/declaremods.mli | 2 -- library/decls.ml | 2 -- library/decls.mli | 2 -- library/dischargedhypsmap.ml | 2 -- library/dischargedhypsmap.mli | 2 -- library/global.ml | 2 -- library/global.mli | 2 -- library/goptions.ml | 2 -- library/goptions.mli | 2 -- library/heads.ml | 2 -- library/heads.mli | 2 -- library/impargs.ml | 2 -- library/impargs.mli | 2 -- library/lib.ml | 2 -- library/lib.mli | 2 -- library/libnames.ml | 2 -- library/libnames.mli | 2 -- library/libobject.ml | 2 -- library/libobject.mli | 2 -- library/library.ml | 2 -- library/library.mli | 2 -- library/nameops.ml | 2 -- library/nameops.mli | 2 -- library/nametab.ml | 2 -- library/nametab.mli | 2 -- library/states.ml | 2 -- library/states.mli | 2 -- library/summary.ml | 2 -- library/summary.mli | 2 -- parsing/argextend.ml4 | 2 -- parsing/egrammar.ml | 2 -- parsing/egrammar.mli | 2 -- parsing/extend.ml | 2 -- parsing/extend.mli | 2 -- parsing/extrawit.ml | 2 -- parsing/extrawit.mli | 2 -- parsing/g_constr.ml4 | 2 -- parsing/g_ltac.ml4 | 2 -- parsing/g_natsyntax.mli | 2 -- parsing/g_prim.ml4 | 2 -- parsing/g_proofs.ml4 | 2 -- parsing/g_tactic.ml4 | 2 -- parsing/g_vernac.ml4 | 2 -- parsing/g_xml.ml4 | 2 -- parsing/g_zsyntax.mli | 2 -- parsing/lexer.ml4 | 2 -- parsing/lexer.mli | 2 -- parsing/pcoq.ml4 | 2 -- parsing/pcoq.mli | 2 -- parsing/ppconstr.ml | 2 -- parsing/ppconstr.mli | 2 -- parsing/pptactic.ml | 2 -- parsing/pptactic.mli | 2 -- parsing/ppvernac.ml | 2 -- parsing/ppvernac.mli | 2 -- parsing/prettyp.ml | 2 -- parsing/prettyp.mli | 2 -- parsing/printer.ml | 2 -- parsing/printer.mli | 2 -- parsing/q_constr.ml4 | 2 -- parsing/q_coqast.ml4 | 2 -- parsing/q_util.ml4 | 2 -- parsing/q_util.mli | 2 -- parsing/tacextend.ml4 | 2 -- parsing/tactic_printer.ml | 2 -- parsing/tactic_printer.mli | 2 -- parsing/vernacextend.ml4 | 2 -- plugins/cc/ccalgo.ml | 2 -- plugins/cc/ccalgo.mli | 2 -- plugins/cc/ccproof.ml | 2 -- plugins/cc/ccproof.mli | 2 -- plugins/cc/cctac.ml | 2 -- plugins/cc/cctac.mli | 2 -- plugins/cc/g_congruence.ml4 | 2 -- plugins/decl_mode/decl_expr.mli | 2 -- plugins/decl_mode/decl_interp.ml | 2 -- plugins/decl_mode/decl_interp.mli | 2 -- plugins/decl_mode/decl_mode.ml | 2 -- plugins/decl_mode/decl_mode.mli | 2 -- plugins/decl_mode/decl_proof_instr.ml | 2 -- plugins/decl_mode/decl_proof_instr.mli | 2 -- plugins/decl_mode/g_decl_mode.ml4 | 2 -- plugins/decl_mode/ppdecl_proof.ml | 2 -- plugins/dp/Dp.v | 2 -- plugins/dp/g_dp.ml4 | 2 -- plugins/dp/zenon.v | 2 -- plugins/extraction/common.ml | 2 -- plugins/extraction/common.mli | 2 -- plugins/extraction/extract_env.ml | 2 -- plugins/extraction/extract_env.mli | 2 -- plugins/extraction/extraction.ml | 2 -- plugins/extraction/extraction.mli | 2 -- plugins/extraction/haskell.ml | 2 -- plugins/extraction/haskell.mli | 2 -- plugins/extraction/miniml.mli | 2 -- plugins/extraction/mlutil.ml | 2 -- plugins/extraction/mlutil.mli | 2 -- plugins/extraction/modutil.ml | 2 -- plugins/extraction/modutil.mli | 2 -- plugins/extraction/ocaml.ml | 2 -- plugins/extraction/ocaml.mli | 2 -- plugins/extraction/scheme.ml | 2 -- plugins/extraction/scheme.mli | 2 -- plugins/extraction/table.ml | 2 -- plugins/extraction/table.mli | 2 -- plugins/field/LegacyField.v | 2 -- plugins/field/LegacyField_Compl.v | 2 -- plugins/field/LegacyField_Tactic.v | 2 -- plugins/field/LegacyField_Theory.v | 2 -- plugins/field/field.ml4 | 2 -- plugins/firstorder/formula.ml | 2 -- plugins/firstorder/formula.mli | 2 -- plugins/firstorder/g_ground.ml4 | 2 -- plugins/firstorder/ground.ml | 2 -- plugins/firstorder/ground.mli | 2 -- plugins/firstorder/instances.ml | 2 -- plugins/firstorder/instances.mli | 2 -- plugins/firstorder/rules.ml | 2 -- plugins/firstorder/rules.mli | 2 -- plugins/firstorder/sequent.ml | 2 -- plugins/firstorder/sequent.mli | 2 -- plugins/firstorder/unify.ml | 2 -- plugins/firstorder/unify.mli | 2 -- plugins/fourier/Fourier.v | 2 -- plugins/fourier/Fourier_util.v | 2 -- plugins/fourier/fourier.ml | 2 -- plugins/fourier/fourierR.ml | 2 -- plugins/fourier/g_fourier.ml4 | 2 -- plugins/funind/merge.ml | 1 - plugins/funind/recdef.ml | 2 -- plugins/micromega/g_micromega.ml4 | 2 -- plugins/omega/Omega.v | 2 -- plugins/omega/OmegaLemmas.v | 2 -- plugins/omega/OmegaPlugin.v | 2 -- plugins/omega/coq_omega.ml | 2 -- plugins/omega/g_omega.ml4 | 2 -- plugins/quote/Quote.v | 2 -- plugins/quote/g_quote.ml4 | 2 -- plugins/quote/quote.ml | 2 -- plugins/ring/LegacyArithRing.v | 2 -- plugins/ring/LegacyNArithRing.v | 2 -- plugins/ring/LegacyRing.v | 2 -- plugins/ring/LegacyRing_theory.v | 2 -- plugins/ring/LegacyZArithRing.v | 2 -- plugins/ring/Ring_abstract.v | 2 -- plugins/ring/Ring_normalize.v | 2 -- plugins/ring/Setoid_ring.v | 2 -- plugins/ring/Setoid_ring_normalize.v | 2 -- plugins/ring/Setoid_ring_theory.v | 2 -- plugins/ring/g_ring.ml4 | 2 -- plugins/ring/ring.ml | 2 -- plugins/rtauto/Bintree.v | 2 -- plugins/rtauto/Rtauto.v | 2 -- plugins/rtauto/g_rtauto.ml4 | 2 -- plugins/rtauto/proof_search.ml | 2 -- plugins/rtauto/proof_search.mli | 2 -- plugins/rtauto/refl_tauto.ml | 2 -- plugins/rtauto/refl_tauto.mli | 2 -- plugins/setoid_ring/newring.ml4 | 2 -- plugins/subtac/eterm.mli | 1 - plugins/subtac/g_subtac.ml4 | 2 -- plugins/subtac/subtac.ml | 2 -- plugins/subtac/subtac_cases.ml | 2 -- plugins/subtac/subtac_cases.mli | 2 -- plugins/subtac/subtac_classes.ml | 2 -- plugins/subtac/subtac_classes.mli | 2 -- plugins/subtac/subtac_coercion.ml | 2 -- plugins/subtac/subtac_pretyping.ml | 2 -- plugins/subtac/subtac_pretyping_F.ml | 2 -- plugins/syntax/ascii_syntax.ml | 2 -- plugins/syntax/nat_syntax.ml | 2 -- plugins/syntax/numbers_syntax.ml | 2 -- plugins/syntax/r_syntax.ml | 2 -- plugins/syntax/string_syntax.ml | 2 -- plugins/syntax/z_syntax.ml | 2 -- plugins/xml/xml.mli | 2 -- plugins/xml/xmlcommand.mli | 2 -- plugins/xml/xmlentries.ml4 | 2 -- pretyping/cases.ml | 2 -- pretyping/cases.mli | 2 -- pretyping/cbv.ml | 2 -- pretyping/cbv.mli | 2 -- pretyping/classops.ml | 2 -- pretyping/classops.mli | 2 -- pretyping/coercion.ml | 2 -- pretyping/coercion.mli | 2 -- pretyping/detyping.ml | 2 -- pretyping/detyping.mli | 2 -- pretyping/evarconv.ml | 2 -- pretyping/evarconv.mli | 2 -- pretyping/evarutil.ml | 2 -- pretyping/evarutil.mli | 2 -- pretyping/evd.ml | 2 -- pretyping/evd.mli | 2 -- pretyping/indrec.ml | 2 -- pretyping/indrec.mli | 2 -- pretyping/inductiveops.ml | 2 -- pretyping/inductiveops.mli | 2 -- pretyping/matching.ml | 2 -- pretyping/matching.mli | 2 -- pretyping/namegen.ml | 2 -- pretyping/namegen.mli | 2 -- pretyping/pattern.ml | 2 -- pretyping/pattern.mli | 2 -- pretyping/pretype_errors.ml | 2 -- pretyping/pretype_errors.mli | 2 -- pretyping/pretyping.ml | 2 -- pretyping/pretyping.mli | 2 -- pretyping/rawterm.ml | 2 -- pretyping/rawterm.mli | 2 -- pretyping/recordops.ml | 2 -- pretyping/recordops.mli | 2 -- pretyping/reductionops.ml | 2 -- pretyping/reductionops.mli | 2 -- pretyping/retyping.ml | 2 -- pretyping/retyping.mli | 2 -- pretyping/tacred.ml | 2 -- pretyping/tacred.mli | 2 -- pretyping/term_dnet.ml | 2 -- pretyping/term_dnet.mli | 2 -- pretyping/termops.ml | 2 -- pretyping/termops.mli | 2 -- pretyping/typeclasses.ml | 2 -- pretyping/typeclasses.mli | 2 -- pretyping/typeclasses_errors.ml | 2 -- pretyping/typeclasses_errors.mli | 2 -- pretyping/typing.ml | 2 -- pretyping/typing.mli | 2 -- pretyping/unification.ml | 2 -- pretyping/unification.mli | 2 -- pretyping/vnorm.ml | 2 -- proofs/clenv.ml | 2 -- proofs/clenv.mli | 2 -- proofs/clenvtac.ml | 2 -- proofs/clenvtac.mli | 2 -- proofs/evar_refiner.ml | 2 -- proofs/evar_refiner.mli | 2 -- proofs/goal.ml | 2 -- proofs/goal.mli | 2 -- proofs/logic.ml | 2 -- proofs/logic.mli | 2 -- proofs/pfedit.ml | 2 -- proofs/pfedit.mli | 2 -- proofs/proof.ml | 2 -- proofs/proof.mli | 2 -- proofs/proof_global.ml | 2 -- proofs/proof_global.mli | 2 -- proofs/proof_type.ml | 2 -- proofs/proof_type.mli | 2 -- proofs/proofview.ml | 2 -- proofs/proofview.mli | 2 -- proofs/redexpr.ml | 2 -- proofs/redexpr.mli | 2 -- proofs/refiner.ml | 2 -- proofs/refiner.mli | 2 -- proofs/tacexpr.ml | 2 -- proofs/tacmach.ml | 2 -- proofs/tacmach.mli | 2 -- proofs/tactic_debug.ml | 2 -- proofs/tactic_debug.mli | 2 -- scripts/coqc.ml | 2 -- scripts/coqmktop.ml | 2 -- tactics/auto.ml | 2 -- tactics/auto.mli | 2 -- tactics/autorewrite.ml | 2 -- tactics/autorewrite.mli | 2 -- tactics/btermdn.ml | 2 -- tactics/btermdn.mli | 2 -- tactics/class_tactics.ml4 | 2 -- tactics/contradiction.ml | 2 -- tactics/contradiction.mli | 2 -- tactics/dhyp.ml | 2 -- tactics/dhyp.mli | 2 -- tactics/eauto.ml4 | 2 -- tactics/elim.ml | 2 -- tactics/elim.mli | 2 -- tactics/elimschemes.ml | 2 -- tactics/elimschemes.mli | 2 -- tactics/eqdecide.ml4 | 2 -- tactics/eqschemes.ml | 2 -- tactics/eqschemes.mli | 2 -- tactics/equality.ml | 2 -- tactics/equality.mli | 2 -- tactics/evar_tactics.ml | 2 -- tactics/evar_tactics.mli | 2 -- tactics/extraargs.ml4 | 2 -- tactics/extraargs.mli | 2 -- tactics/extratactics.ml4 | 2 -- tactics/extratactics.mli | 2 -- tactics/hiddentac.ml | 2 -- tactics/hiddentac.mli | 2 -- tactics/hipattern.ml4 | 2 -- tactics/hipattern.mli | 2 -- tactics/inv.ml | 2 -- tactics/inv.mli | 2 -- tactics/leminv.ml | 2 -- tactics/nbtermdn.ml | 2 -- tactics/nbtermdn.mli | 2 -- tactics/refine.ml | 2 -- tactics/refine.mli | 2 -- tactics/rewrite.ml4 | 2 -- tactics/tacinterp.ml | 2 -- tactics/tacinterp.mli | 2 -- tactics/tactic_option.ml | 2 -- tactics/tactic_option.mli | 2 -- tactics/tacticals.ml | 2 -- tactics/tacticals.mli | 2 -- tactics/tactics.ml | 2 -- tactics/tactics.mli | 2 -- tactics/tauto.ml4 | 2 -- tactics/termdn.ml | 2 -- tactics/termdn.mli | 2 -- test-suite/bugs/closed/shouldsucceed/1507.v | 1 - test-suite/misc/berardi_test.v | 2 -- test-suite/success/Field.v | 2 -- test-suite/success/LegacyField.v | 2 -- test-suite/success/Tauto.v | 2 -- test-suite/typeclasses/NewSetoid.v | 2 -- theories/Arith/Arith.v | 2 -- theories/Arith/Arith_base.v | 2 -- theories/Arith/Between.v | 2 -- theories/Arith/Bool_nat.v | 2 -- theories/Arith/Compare.v | 2 -- theories/Arith/Compare_dec.v | 2 -- theories/Arith/Div2.v | 2 -- theories/Arith/EqNat.v | 2 -- theories/Arith/Euclid.v | 2 -- theories/Arith/Even.v | 2 -- theories/Arith/Factorial.v | 2 -- theories/Arith/Gt.v | 2 -- theories/Arith/Le.v | 2 -- theories/Arith/Lt.v | 2 -- theories/Arith/Max.v | 2 -- theories/Arith/Min.v | 2 -- theories/Arith/Minus.v | 2 -- theories/Arith/Mult.v | 2 -- theories/Arith/Peano_dec.v | 2 -- theories/Arith/Plus.v | 2 -- theories/Arith/Wf_nat.v | 2 -- theories/Bool/Bool.v | 2 -- theories/Bool/BoolEq.v | 1 - theories/Bool/Bvector.v | 2 -- theories/Bool/DecBool.v | 2 -- theories/Bool/IfProp.v | 2 -- theories/Bool/Sumbool.v | 2 -- theories/Bool/Zerob.v | 2 -- theories/Classes/EquivDec.v | 2 -- theories/Classes/Equivalence.v | 2 -- theories/Classes/Init.v | 2 -- theories/Classes/Morphisms.v | 2 -- theories/Classes/RelationClasses.v | 2 -- theories/Classes/SetoidClass.v | 2 -- theories/Classes/SetoidDec.v | 2 -- theories/Classes/SetoidTactics.v | 2 -- theories/FSets/FMapAVL.v | 2 -- theories/FSets/FMapFacts.v | 2 -- theories/FSets/FMapFullAVL.v | 2 -- theories/FSets/FMapInterface.v | 2 -- theories/FSets/FMapList.v | 2 -- theories/FSets/FMapPositive.v | 2 -- theories/FSets/FMapWeakList.v | 2 -- theories/FSets/FMaps.v | 2 -- theories/FSets/FSetAVL.v | 2 -- theories/FSets/FSetBridge.v | 2 -- theories/FSets/FSetDecide.v | 2 -- theories/FSets/FSetEqProperties.v | 2 -- theories/FSets/FSetFacts.v | 2 -- theories/FSets/FSetInterface.v | 2 -- theories/FSets/FSetList.v | 2 -- theories/FSets/FSetProperties.v | 2 -- theories/FSets/FSetToFiniteSet.v | 2 -- theories/FSets/FSetWeakList.v | 2 -- theories/FSets/FSets.v | 2 -- theories/Init/Datatypes.v | 2 -- theories/Init/Logic.v | 2 -- theories/Init/Logic_Type.v | 2 -- theories/Init/Notations.v | 2 -- theories/Init/Peano.v | 2 -- theories/Init/Prelude.v | 2 -- theories/Init/Specif.v | 2 -- theories/Init/Tactics.v | 2 -- theories/Init/Wf.v | 2 -- theories/Lists/List.v | 2 -- theories/Lists/ListSet.v | 2 -- theories/Lists/ListTactics.v | 2 -- theories/Lists/SetoidList.v | 2 -- theories/Lists/Streams.v | 2 -- theories/Lists/TheoryList.v | 2 -- theories/Logic/Berardi.v | 2 -- theories/Logic/ChoiceFacts.v | 2 -- theories/Logic/Classical.v | 2 -- theories/Logic/ClassicalChoice.v | 2 -- theories/Logic/ClassicalDescription.v | 2 -- theories/Logic/ClassicalEpsilon.v | 2 -- theories/Logic/ClassicalFacts.v | 2 -- theories/Logic/ClassicalUniqueChoice.v | 2 -- theories/Logic/Classical_Pred_Set.v | 2 -- theories/Logic/Classical_Pred_Type.v | 2 -- theories/Logic/Classical_Prop.v | 2 -- theories/Logic/Classical_Type.v | 2 -- theories/Logic/ConstructiveEpsilon.v | 2 -- theories/Logic/Decidable.v | 2 -- theories/Logic/Description.v | 2 -- theories/Logic/Diaconescu.v | 2 -- theories/Logic/Epsilon.v | 2 -- theories/Logic/Eqdep.v | 2 -- theories/Logic/EqdepFacts.v | 2 -- theories/Logic/Eqdep_dec.v | 2 -- theories/Logic/FunctionalExtensionality.v | 2 -- theories/Logic/IndefiniteDescription.v | 2 -- theories/Logic/JMeq.v | 2 -- theories/Logic/RelationalChoice.v | 2 -- theories/MSets/MSetAVL.v | 2 -- theories/MSets/MSetDecide.v | 2 -- theories/MSets/MSetEqProperties.v | 2 -- theories/MSets/MSetFacts.v | 2 -- theories/MSets/MSetInterface.v | 2 -- theories/MSets/MSetList.v | 2 -- theories/MSets/MSetProperties.v | 2 -- theories/MSets/MSetToFiniteSet.v | 2 -- theories/MSets/MSetWeakList.v | 2 -- theories/MSets/MSets.v | 2 -- theories/NArith/BinNat.v | 2 -- theories/NArith/BinPos.v | 2 -- theories/NArith/NArith.v | 2 -- theories/NArith/Ndec.v | 2 -- theories/NArith/Ndigits.v | 2 -- theories/NArith/Ndist.v | 2 -- theories/NArith/Nnat.v | 2 -- theories/NArith/Pnat.v | 2 -- theories/Numbers/BigNumPrelude.v | 2 -- theories/Numbers/Cyclic/Abstract/CyclicAxioms.v | 2 -- theories/Numbers/Cyclic/Abstract/NZCyclic.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleAdd.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleBase.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleCyclic.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleDiv.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleDivn1.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleLift.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleMul.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleSqrt.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleSub.v | 2 -- theories/Numbers/Cyclic/DoubleCyclic/DoubleType.v | 2 -- theories/Numbers/Cyclic/Int31/Cyclic31.v | 2 -- theories/Numbers/Cyclic/Int31/Int31.v | 2 -- theories/Numbers/Cyclic/Int31/Ring31.v | 2 -- theories/Numbers/Cyclic/ZModulo/ZModulo.v | 2 -- theories/Numbers/Integer/Abstract/ZAdd.v | 2 -- theories/Numbers/Integer/Abstract/ZAddOrder.v | 2 -- theories/Numbers/Integer/Abstract/ZAxioms.v | 2 -- theories/Numbers/Integer/Abstract/ZBase.v | 2 -- theories/Numbers/Integer/Abstract/ZLt.v | 2 -- theories/Numbers/Integer/Abstract/ZMul.v | 2 -- theories/Numbers/Integer/Abstract/ZMulOrder.v | 2 -- theories/Numbers/Integer/Abstract/ZProperties.v | 2 -- theories/Numbers/Integer/BigZ/BigZ.v | 2 -- theories/Numbers/Integer/BigZ/ZMake.v | 2 -- theories/Numbers/Integer/Binary/ZBinary.v | 2 -- theories/Numbers/Integer/NatPairs/ZNatPairs.v | 2 -- theories/Numbers/Integer/SpecViaZ/ZSig.v | 2 -- theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v | 2 -- theories/Numbers/NaryFunctions.v | 2 -- theories/Numbers/NatInt/NZAdd.v | 2 -- theories/Numbers/NatInt/NZAddOrder.v | 2 -- theories/Numbers/NatInt/NZAxioms.v | 2 -- theories/Numbers/NatInt/NZBase.v | 2 -- theories/Numbers/NatInt/NZDomain.v | 2 -- theories/Numbers/NatInt/NZMul.v | 2 -- theories/Numbers/NatInt/NZMulOrder.v | 2 -- theories/Numbers/NatInt/NZOrder.v | 2 -- theories/Numbers/NatInt/NZProperties.v | 2 -- theories/Numbers/Natural/Abstract/NAdd.v | 2 -- theories/Numbers/Natural/Abstract/NAddOrder.v | 2 -- theories/Numbers/Natural/Abstract/NAxioms.v | 2 -- theories/Numbers/Natural/Abstract/NBase.v | 2 -- theories/Numbers/Natural/Abstract/NDefOps.v | 2 -- theories/Numbers/Natural/Abstract/NIso.v | 2 -- theories/Numbers/Natural/Abstract/NMulOrder.v | 2 -- theories/Numbers/Natural/Abstract/NOrder.v | 2 -- theories/Numbers/Natural/Abstract/NProperties.v | 2 -- theories/Numbers/Natural/Abstract/NStrongRec.v | 2 -- theories/Numbers/Natural/Abstract/NSub.v | 2 -- theories/Numbers/Natural/BigN/NMake_gen.ml | 2 -- theories/Numbers/Natural/BigN/Nbasic.v | 2 -- theories/Numbers/Natural/Binary/NBinary.v | 2 -- theories/Numbers/Natural/Peano/NPeano.v | 2 -- theories/Numbers/Natural/SpecViaZ/NSig.v | 2 -- theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v | 2 -- theories/Numbers/NumPrelude.v | 2 -- theories/Numbers/Rational/SpecViaQ/QSig.v | 2 -- theories/Program/Basics.v | 2 -- theories/Program/Combinators.v | 2 -- theories/Program/Equality.v | 2 -- theories/Program/Program.v | 2 -- theories/Program/Subset.v | 2 -- theories/Program/Syntax.v | 2 -- theories/Program/Tactics.v | 2 -- theories/Program/Utils.v | 2 -- theories/Program/Wf.v | 2 -- theories/QArith/QArith.v | 2 -- theories/QArith/QArith_base.v | 2 -- theories/QArith/Qcanon.v | 2 -- theories/QArith/Qfield.v | 2 -- theories/QArith/Qreals.v | 2 -- theories/QArith/Qreduction.v | 2 -- theories/QArith/Qring.v | 2 -- theories/Reals/Alembert.v | 2 -- theories/Reals/AltSeries.v | 2 -- theories/Reals/ArithProp.v | 2 -- theories/Reals/Binomial.v | 2 -- theories/Reals/Cauchy_prod.v | 2 -- theories/Reals/Cos_plus.v | 2 -- theories/Reals/Cos_rel.v | 2 -- theories/Reals/DiscrR.v | 2 -- theories/Reals/Exp_prop.v | 2 -- theories/Reals/Integration.v | 2 -- theories/Reals/LegacyRfield.v | 2 -- theories/Reals/MVT.v | 2 -- theories/Reals/NewtonInt.v | 2 -- theories/Reals/PSeries_reg.v | 2 -- theories/Reals/PartSum.v | 2 -- theories/Reals/RIneq.v | 2 -- theories/Reals/RList.v | 2 -- theories/Reals/R_Ifp.v | 2 -- theories/Reals/R_sqr.v | 2 -- theories/Reals/R_sqrt.v | 2 -- theories/Reals/Ranalysis.v | 2 -- theories/Reals/Ranalysis1.v | 2 -- theories/Reals/Ranalysis2.v | 2 -- theories/Reals/Ranalysis3.v | 2 -- theories/Reals/Ranalysis4.v | 2 -- theories/Reals/Raxioms.v | 2 -- theories/Reals/Rbase.v | 2 -- theories/Reals/Rbasic_fun.v | 2 -- theories/Reals/Rcomplete.v | 2 -- theories/Reals/Rdefinitions.v | 2 -- theories/Reals/Rderiv.v | 2 -- theories/Reals/Reals.v | 2 -- theories/Reals/Rfunctions.v | 2 -- theories/Reals/Rgeom.v | 2 -- theories/Reals/RiemannInt.v | 2 -- theories/Reals/RiemannInt_SF.v | 2 -- theories/Reals/Rlimit.v | 2 -- theories/Reals/Rpow_def.v | 2 -- theories/Reals/Rpower.v | 1 - theories/Reals/Rprod.v | 2 -- theories/Reals/Rseries.v | 2 -- theories/Reals/Rsigma.v | 2 -- theories/Reals/Rsqrt_def.v | 2 -- theories/Reals/Rtopology.v | 2 -- theories/Reals/Rtrigo.v | 2 -- theories/Reals/Rtrigo_alt.v | 2 -- theories/Reals/Rtrigo_calc.v | 2 -- theories/Reals/Rtrigo_def.v | 2 -- theories/Reals/Rtrigo_fun.v | 2 -- theories/Reals/Rtrigo_reg.v | 2 -- theories/Reals/SeqProp.v | 2 -- theories/Reals/SeqSeries.v | 2 -- theories/Reals/SplitAbsolu.v | 2 -- theories/Reals/SplitRmult.v | 2 -- theories/Reals/Sqrt_reg.v | 2 -- theories/Relations/Operators_Properties.v | 2 -- theories/Relations/Relation_Definitions.v | 2 -- theories/Relations/Relation_Operators.v | 2 -- theories/Relations/Relations.v | 2 -- theories/Setoids/Setoid.v | 2 -- theories/Sets/Classical_sets.v | 2 -- theories/Sets/Constructive_sets.v | 2 -- theories/Sets/Cpo.v | 2 -- theories/Sets/Ensembles.v | 2 -- theories/Sets/Finite_sets.v | 2 -- theories/Sets/Finite_sets_facts.v | 2 -- theories/Sets/Image.v | 2 -- theories/Sets/Infinite_sets.v | 2 -- theories/Sets/Integers.v | 2 -- theories/Sets/Multiset.v | 2 -- theories/Sets/Partial_Order.v | 2 -- theories/Sets/Permut.v | 2 -- theories/Sets/Powerset.v | 2 -- theories/Sets/Powerset_Classical_facts.v | 2 -- theories/Sets/Powerset_facts.v | 2 -- theories/Sets/Relations_1.v | 2 -- theories/Sets/Relations_1_facts.v | 2 -- theories/Sets/Relations_2.v | 2 -- theories/Sets/Relations_2_facts.v | 2 -- theories/Sets/Relations_3.v | 2 -- theories/Sets/Relations_3_facts.v | 2 -- theories/Sets/Uniset.v | 2 -- theories/Sorting/Heap.v | 2 -- theories/Sorting/Mergesort.v | 2 -- theories/Sorting/PermutEq.v | 2 -- theories/Sorting/PermutSetoid.v | 2 -- theories/Sorting/Permutation.v | 2 -- theories/Sorting/Sorted.v | 2 -- theories/Sorting/Sorting.v | 2 -- theories/Strings/Ascii.v | 2 -- theories/Strings/String.v | 2 -- theories/Structures/DecidableType.v | 2 -- theories/Structures/DecidableTypeEx.v | 2 -- theories/Structures/Equalities.v | 2 -- theories/Structures/OrderedType.v | 2 -- theories/Structures/OrderedTypeAlt.v | 2 -- theories/Structures/OrderedTypeEx.v | 2 -- theories/Structures/Orders.v | 2 -- theories/Structures/OrdersAlt.v | 2 -- theories/Structures/OrdersEx.v | 2 -- theories/Wellfounded/Disjoint_Union.v | 2 -- theories/Wellfounded/Inclusion.v | 2 -- theories/Wellfounded/Inverse_Image.v | 2 -- theories/Wellfounded/Lexicographic_Exponentiation.v | 2 -- theories/Wellfounded/Lexicographic_Product.v | 2 -- theories/Wellfounded/Transitive_Closure.v | 2 -- theories/Wellfounded/Union.v | 2 -- theories/Wellfounded/Well_Ordering.v | 2 -- theories/Wellfounded/Wellfounded.v | 2 -- theories/ZArith/BinInt.v | 2 -- theories/ZArith/Int.v | 2 -- theories/ZArith/Wf_Z.v | 2 -- theories/ZArith/ZArith.v | 2 -- theories/ZArith/ZArith_base.v | 2 -- theories/ZArith/ZArith_dec.v | 2 -- theories/ZArith/Zabs.v | 2 -- theories/ZArith/Zbool.v | 2 -- theories/ZArith/Zcomplements.v | 2 -- theories/ZArith/Zdigits.v | 2 -- theories/ZArith/Zdiv.v | 2 -- theories/ZArith/Zeven.v | 2 -- theories/ZArith/Zgcd_alt.v | 2 -- theories/ZArith/Zhints.v | 2 -- theories/ZArith/Zlogarithm.v | 2 -- theories/ZArith/Zmax.v | 2 -- theories/ZArith/Zmin.v | 2 -- theories/ZArith/Zmisc.v | 2 -- theories/ZArith/Znat.v | 2 -- theories/ZArith/Znumtheory.v | 2 -- theories/ZArith/Zorder.v | 2 -- theories/ZArith/Zpow_facts.v | 2 -- theories/ZArith/Zpower.v | 2 -- theories/ZArith/Zsqrt.v | 2 -- theories/ZArith/Zwf.v | 2 -- theories/ZArith/auxiliary.v | 2 -- tools/coq_makefile.ml4 | 2 -- tools/coq_tex.ml4 | 2 -- tools/coqdep.ml | 2 -- tools/coqdep_boot.ml | 2 -- tools/coqdep_common.ml | 2 -- tools/coqdep_lexer.mll | 2 -- tools/coqdoc/alpha.ml | 2 -- tools/coqdoc/alpha.mli | 2 -- tools/coqdoc/cpretty.mli | 2 -- tools/coqdoc/cpretty.mll | 2 -- tools/coqdoc/index.ml | 2 -- tools/coqdoc/index.mli | 2 -- tools/coqdoc/main.ml | 2 -- tools/coqdoc/output.ml | 2 -- tools/coqdoc/output.mli | 2 -- tools/coqwc.mll | 2 -- tools/gallina.ml | 2 -- tools/gallina_lexer.mll | 2 -- toplevel/auto_ind_decl.ml | 2 -- toplevel/autoinstance.ml | 2 -- toplevel/cerrors.ml | 2 -- toplevel/cerrors.mli | 2 -- toplevel/class.ml | 2 -- toplevel/class.mli | 2 -- toplevel/classes.ml | 2 -- toplevel/classes.mli | 2 -- toplevel/command.ml | 2 -- toplevel/command.mli | 2 -- toplevel/coqinit.ml | 2 -- toplevel/coqinit.mli | 2 -- toplevel/coqtop.ml | 2 -- toplevel/coqtop.mli | 2 -- toplevel/discharge.ml | 2 -- toplevel/discharge.mli | 2 -- toplevel/himsg.ml | 2 -- toplevel/himsg.mli | 2 -- toplevel/ind_tables.ml | 2 -- toplevel/indschemes.ml | 2 -- toplevel/indschemes.mli | 2 -- toplevel/lemmas.ml | 2 -- toplevel/lemmas.mli | 2 -- toplevel/metasyntax.ml | 2 -- toplevel/metasyntax.mli | 2 -- toplevel/mltop.ml4 | 2 -- toplevel/mltop.mli | 2 -- toplevel/record.ml | 2 -- toplevel/record.mli | 2 -- toplevel/search.ml | 2 -- toplevel/search.mli | 2 -- toplevel/toplevel.ml | 2 -- toplevel/toplevel.mli | 2 -- toplevel/usage.ml | 2 -- toplevel/usage.mli | 2 -- toplevel/vernac.ml | 2 -- toplevel/vernac.mli | 2 -- toplevel/vernacentries.ml | 2 -- toplevel/vernacentries.mli | 2 -- toplevel/vernacexpr.ml | 2 -- toplevel/vernacinterp.ml | 2 -- toplevel/vernacinterp.mli | 2 -- toplevel/whelp.ml4 | 2 -- toplevel/whelp.mli | 2 -- 901 files changed, 1789 deletions(-) diff --git a/Makefile b/Makefile index 3011e7d00..f1f04e77d 100644 --- a/Makefile +++ b/Makefile @@ -6,8 +6,6 @@ # # GNU Lesser General Public License Version 2.1 # ####################################################################### -# $Id$ - # Makefile for Coq # diff --git a/Makefile.build b/Makefile.build index 8ded28301..fe2bba29e 100644 --- a/Makefile.build +++ b/Makefile.build @@ -6,8 +6,6 @@ # # GNU Lesser General Public License Version 2.1 # ####################################################################### -# $Id$ - # This makefile is normally called by the main Makefile after setting # some variables. diff --git a/checker/check.ml b/checker/check.ml index 0a75f0137..0317416f3 100644 --- a/checker/check.ml +++ b/checker/check.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: library.ml 9679 2007-02-24 15:22:07Z herbelin $ *) - open Pp open Util open Names diff --git a/checker/checker.ml b/checker/checker.ml index e15c37e67..9489dc94b 100644 --- a/checker/checker.ml +++ b/checker/checker.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: coqtop.ml 10153 2007-09-28 18:00:45Z glondu $ *) - open Pp open Util open System diff --git a/checker/closure.ml b/checker/closure.ml index c710df816..054057d1f 100644 --- a/checker/closure.ml +++ b/checker/closure.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: closure.ml 9983 2007-07-12 17:15:22Z barras $ *) - open Util open Pp open Term diff --git a/checker/closure.mli b/checker/closure.mli index 260d159b3..ada7ded1e 100644 --- a/checker/closure.mli +++ b/checker/closure.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: closure.mli 9902 2007-06-21 17:01:21Z herbelin $ i*) - (*i*) open Pp open Names diff --git a/checker/indtypes.ml b/checker/indtypes.ml index de57c50a7..0b4c6fde3 100644 --- a/checker/indtypes.ml +++ b/checker/indtypes.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: indtypes.ml 10296 2007-11-07 11:02:42Z barras $ *) - open Util open Names open Univ diff --git a/checker/indtypes.mli b/checker/indtypes.mli index b920315ab..12511df33 100644 --- a/checker/indtypes.mli +++ b/checker/indtypes.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: indtypes.mli 9831 2007-05-17 18:55:42Z herbelin $ i*) - (*i*) open Names open Univ diff --git a/checker/inductive.ml b/checker/inductive.ml index 4faf99a90..54bf1bbe6 100644 --- a/checker/inductive.ml +++ b/checker/inductive.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: inductive.ml 10172 2007-10-04 13:02:03Z herbelin $ *) - open Util open Names open Univ diff --git a/checker/inductive.mli b/checker/inductive.mli index 8e6d4ffb9..bd758772a 100644 --- a/checker/inductive.mli +++ b/checker/inductive.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: inductive.mli 9420 2006-12-08 15:34:09Z barras $ i*) - (*i*) open Names open Term diff --git a/checker/modops.ml b/checker/modops.ml index ce2f07ab6..e6428d5ab 100644 --- a/checker/modops.ml +++ b/checker/modops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: modops.ml 9872 2007-05-30 16:01:18Z soubiran $ i*) - (*i*) open Util open Pp diff --git a/checker/modops.mli b/checker/modops.mli index 4476013c6..fedcf32cb 100644 --- a/checker/modops.mli +++ b/checker/modops.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: modops.mli 9821 2007-05-11 17:00:58Z aspiwack $ i*) - (*i*) open Util open Names diff --git a/checker/reduction.ml b/checker/reduction.ml index 612e7562f..776edb243 100644 --- a/checker/reduction.ml +++ b/checker/reduction.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: reduction.ml 9215 2006-10-05 15:40:31Z herbelin $ *) - open Util open Names open Term diff --git a/checker/reduction.mli b/checker/reduction.mli index 81c93ee53..02b856edc 100644 --- a/checker/reduction.mli +++ b/checker/reduction.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: reduction.mli 7639 2005-12-02 10:01:15Z gregoire $ i*) - (*i*) open Term open Environ diff --git a/checker/safe_typing.ml b/checker/safe_typing.ml index 98534e08c..e37ff370c 100644 --- a/checker/safe_typing.ml +++ b/checker/safe_typing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: safe_typing.ml 10275 2007-10-30 11:01:24Z barras $ *) - open Pp open Util open Names diff --git a/checker/safe_typing.mli b/checker/safe_typing.mli index 12fdbfce8..ded3fe47f 100644 --- a/checker/safe_typing.mli +++ b/checker/safe_typing.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: safe_typing.mli 9821 2007-05-11 17:00:58Z aspiwack $ i*) - (*i*) open Names open Term diff --git a/checker/subtyping.ml b/checker/subtyping.ml index ec1c908a6..9df49630c 100644 --- a/checker/subtyping.ml +++ b/checker/subtyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: subtyping.ml 10664 2008-03-14 11:27:37Z soubiran $ i*) - (*i*) open Util open Names diff --git a/checker/subtyping.mli b/checker/subtyping.mli index 10842252e..1b0ca5c16 100644 --- a/checker/subtyping.mli +++ b/checker/subtyping.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: subtyping.mli 5920 2004-07-16 20:01:26Z herbelin $ i*) - (*i*) open Univ open Term diff --git a/checker/term.ml b/checker/term.ml index 35ae1121e..8d65bbe17 100644 --- a/checker/term.ml +++ b/checker/term.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: term.ml 10098 2007-08-27 11:41:08Z herbelin $ *) - (* This module instantiates the structure of generic deBruijn terms to Coq *) open Util diff --git a/checker/type_errors.ml b/checker/type_errors.ml index 7c0141055..bddda852d 100644 --- a/checker/type_errors.ml +++ b/checker/type_errors.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: type_errors.ml 8845 2006-05-23 07:41:58Z herbelin $ *) - open Names open Term open Environ diff --git a/checker/type_errors.mli b/checker/type_errors.mli index 0482f2f2a..70971faa4 100644 --- a/checker/type_errors.mli +++ b/checker/type_errors.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: type_errors.mli 8845 2006-05-23 07:41:58Z herbelin $ i*) - (*i*) open Names open Term diff --git a/checker/typeops.ml b/checker/typeops.ml index e5cf6a6d6..1007c8971 100644 --- a/checker/typeops.ml +++ b/checker/typeops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: typeops.ml 9314 2006-10-29 20:11:08Z herbelin $ *) - open Util open Names open Univ diff --git a/checker/typeops.mli b/checker/typeops.mli index de160a79b..d554af026 100644 --- a/checker/typeops.mli +++ b/checker/typeops.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: typeops.mli 9427 2006-12-11 18:46:35Z bgregoir $ i*) - (*i*) open Names open Term diff --git a/checker/validate.ml b/checker/validate.ml index ab17aa7f8..d3d2ecb60 100644 --- a/checker/validate.ml +++ b/checker/validate.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This module defines validation functions to ensure an imported value (using input_value) has the correct structure. *) diff --git a/config/coq_config.mli b/config/coq_config.mli index 2cd1e4543..1a83ca54c 100644 --- a/config/coq_config.mli +++ b/config/coq_config.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val local : bool (* local use (no installation) *) val coqlib : string (* where the std library is installed *) diff --git a/configure b/configure index fc77ee10c..5ad950260 100755 --- a/configure +++ b/configure @@ -1106,4 +1106,3 @@ echo echo "*Warning* To compile the system for a new architecture" echo " don't forget to do a 'make archclean' before './configure'." -# $Id$ diff --git a/doc/common/macros.tex b/doc/common/macros.tex index 6048a75fd..c4e797363 100755 --- a/doc/common/macros.tex +++ b/doc/common/macros.tex @@ -520,8 +520,6 @@ {\begin{center}\begin{rulebox}} {\end{rulebox}\end{center}} -% $Id$ - %%% Local Variables: %%% mode: latex diff --git a/doc/common/title.tex b/doc/common/title.tex index abd106ea4..1dc524324 100755 --- a/doc/common/title.tex +++ b/doc/common/title.tex @@ -70,4 +70,3 @@ V\coqversion, \today % TeX-master: "" % End: -% $Id$ diff --git a/doc/refman/Extraction.tex b/doc/refman/Extraction.tex index cfc943413..277e3d539 100644 --- a/doc/refman/Extraction.tex +++ b/doc/refman/Extraction.tex @@ -684,8 +684,6 @@ of the sources of \Coq. After compilation those two examples run nonetheless, thanks to the correction of the extraction~\cite{Let02}. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-add.tex b/doc/refman/RefMan-add.tex index 52746fad6..2094c9d2d 100644 --- a/doc/refman/RefMan-add.tex +++ b/doc/refman/RefMan-add.tex @@ -51,8 +51,6 @@ can be found in the document {\tt Polynom.dvi} %anomalous behavior, please check first whether it has been already %reported in this document. -% $Id$ - %%% Local Variables: %%% mode: latex diff --git a/doc/refman/RefMan-cic.tex b/doc/refman/RefMan-cic.tex index f50c4fe1f..4d473d54b 100644 --- a/doc/refman/RefMan-cic.tex +++ b/doc/refman/RefMan-cic.tex @@ -1706,8 +1706,6 @@ impredicative system for sort \Set{} become~: -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-coi.tex b/doc/refman/RefMan-coi.tex index 2c0396642..619a8ee10 100644 --- a/doc/refman/RefMan-coi.tex +++ b/doc/refman/RefMan-coi.tex @@ -403,4 +403,3 @@ See \cite{Gimenez95b} for a complete description about this development. %\end{document} -% $Id$ diff --git a/doc/refman/RefMan-com.tex b/doc/refman/RefMan-com.tex index cf4774285..824943d47 100644 --- a/doc/refman/RefMan-com.tex +++ b/doc/refman/RefMan-com.tex @@ -376,8 +376,6 @@ makes more disk access. It is also less secure since an attacker might have replaced the compiled library $A$ after it has been read by the first command, but before it has been read by the second command. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-gal.tex b/doc/refman/RefMan-gal.tex index 974106164..5461779fe 100644 --- a/doc/refman/RefMan-gal.tex +++ b/doc/refman/RefMan-gal.tex @@ -1657,4 +1657,3 @@ To be able to unfold a proof, you should end the proof by {\tt Defined} % TeX-master: "Reference-Manual" % End: -% $Id$ diff --git a/doc/refman/RefMan-ide.tex b/doc/refman/RefMan-ide.tex index 831eb9d08..c00a389f4 100644 --- a/doc/refman/RefMan-ide.tex +++ b/doc/refman/RefMan-ide.tex @@ -312,8 +312,6 @@ or -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-ind.tex b/doc/refman/RefMan-ind.tex index 23006b72e..959442402 100644 --- a/doc/refman/RefMan-ind.tex +++ b/doc/refman/RefMan-ind.tex @@ -508,4 +508,3 @@ Check tree_forest_mutind. %\end{document} -% $Id$ diff --git a/doc/refman/RefMan-int.tex b/doc/refman/RefMan-int.tex index c40224a48..6d2c37f75 100644 --- a/doc/refman/RefMan-int.tex +++ b/doc/refman/RefMan-int.tex @@ -140,8 +140,6 @@ is given in the additional document {\tt Library.ps}. \end{description} -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-lib.tex b/doc/refman/RefMan-lib.tex index 99c25d056..7caf6126e 100644 --- a/doc/refman/RefMan-lib.tex +++ b/doc/refman/RefMan-lib.tex @@ -1095,8 +1095,6 @@ description, etc.) and the possibility to download them one by one. You will also find informations on how to submit a new contribution. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-modr.tex b/doc/refman/RefMan-modr.tex index 05bc3496e..9ab8aded9 100644 --- a/doc/refman/RefMan-modr.tex +++ b/doc/refman/RefMan-modr.tex @@ -556,8 +556,6 @@ In the rules below we assume $\Gamma_P$ is $[p_1:P_1;\ldots;p_r:P_r]$, % \end{itemize} -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-oth.tex b/doc/refman/RefMan-oth.tex index 9e18d0af2..b765ef7d4 100644 --- a/doc/refman/RefMan-oth.tex +++ b/doc/refman/RefMan-oth.tex @@ -1121,8 +1121,6 @@ control the scope of their effect. There are four kinds of commands: \end{itemize} -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-pre.tex b/doc/refman/RefMan-pre.tex index 1b6efc582..736627122 100644 --- a/doc/refman/RefMan-pre.tex +++ b/doc/refman/RefMan-pre.tex @@ -698,8 +698,6 @@ Hugo Herbelin\\ % Integration of ZArith lemmas from Sophia and Nijmegen. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-pro.tex b/doc/refman/RefMan-pro.tex index 593ed771f..a8bb7966a 100644 --- a/doc/refman/RefMan-pro.tex +++ b/doc/refman/RefMan-pro.tex @@ -402,8 +402,6 @@ All the hypotheses remains usable in the proof development. This command goes back to the default mode which is to print all available hypotheses. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-syn.tex b/doc/refman/RefMan-syn.tex index 548c25985..6b471ec39 100644 --- a/doc/refman/RefMan-syn.tex +++ b/doc/refman/RefMan-syn.tex @@ -1101,8 +1101,6 @@ places where a list of the underlying entry can be used: {\nterm{entry}} is either {\tt\small constr}, {\tt\small hyp}, {\tt\small integer} or {\tt\small int\_or\_var}. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-tac.tex b/doc/refman/RefMan-tac.tex index 139f80cf3..0e6bff9db 100644 --- a/doc/refman/RefMan-tac.tex +++ b/doc/refman/RefMan-tac.tex @@ -4257,8 +4257,6 @@ Chapter~\ref{TacticLanguage} gives examples of more complex user-defined tactics. -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: "Reference-Manual" diff --git a/doc/refman/RefMan-uti.tex b/doc/refman/RefMan-uti.tex index f1dde04ad..996a15cd4 100644 --- a/doc/refman/RefMan-uti.tex +++ b/doc/refman/RefMan-uti.tex @@ -264,8 +264,6 @@ There are man pages for the commands {\tt coqdep}, {\tt gallina} and \RefManCutCommand{ENDREFMAN=\thepage} %END LATEX -% $Id$ - %%% Local Variables: %%% mode: latex %%% TeX-master: t diff --git a/doc/refman/Reference-Manual.tex b/doc/refman/Reference-Manual.tex index 946bfda12..0c90e61ba 100644 --- a/doc/refman/Reference-Manual.tex +++ b/doc/refman/Reference-Manual.tex @@ -138,4 +138,3 @@ Options A and B of the licence are {\em not} elected.} \end{document} -% $Id$ diff --git a/doc/stdlib/Library.tex b/doc/stdlib/Library.tex index f5509c3a3..02dc61bfe 100755 --- a/doc/stdlib/Library.tex +++ b/doc/stdlib/Library.tex @@ -61,4 +61,3 @@ you can access from the \Coq\ home page at \end{document} -% $Id$ diff --git a/doc/tutorial/Tutorial.tex b/doc/tutorial/Tutorial.tex index 219706e35..43c8bf620 100755 --- a/doc/tutorial/Tutorial.tex +++ b/doc/tutorial/Tutorial.tex @@ -1574,4 +1574,3 @@ with \Coq, in order to acquaint yourself with various proof techniques. \end{document} -% $Id$ diff --git a/ide/command_windows.ml b/ide/command_windows.ml index f6ef42221..92dcd8222 100644 --- a/ide/command_windows.ml +++ b/ide/command_windows.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - class command_window () = (* let window = GWindow.window ~allow_grow:true ~allow_shrink:true diff --git a/ide/command_windows.mli b/ide/command_windows.mli index 4104f086c..b211afabd 100644 --- a/ide/command_windows.mli +++ b/ide/command_windows.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - class command_window : unit -> object diff --git a/ide/config_lexer.mll b/ide/config_lexer.mll index 97aeb2f5a..cafa96e43 100644 --- a/ide/config_lexer.mll +++ b/ide/config_lexer.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - { open Lexing diff --git a/ide/config_parser.mly b/ide/config_parser.mly index bd5577db3..104d31f3c 100644 --- a/ide/config_parser.mly +++ b/ide/config_parser.mly @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************/ -/* $Id$ */ - %{ open Parsing diff --git a/ide/coq.ml b/ide/coq.ml index 9b0afc7be..383a7a34c 100644 --- a/ide/coq.ml +++ b/ide/coq.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Vernac open Vernacexpr open Pfedit diff --git a/ide/coq.mli b/ide/coq.mli index d30f7168f..d1568203f 100644 --- a/ide/coq.mli +++ b/ide/coq.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/ide/coq_commands.ml b/ide/coq_commands.ml index e4a3ae56a..1d56489df 100644 --- a/ide/coq_commands.ml +++ b/ide/coq_commands.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - let commands = [ [(* "Abort"; *) "Add Abstract Ring A Aplus Amult Aone Azero Ainv Aeq T."; diff --git a/ide/coq_lex.mll b/ide/coq_lex.mll index 36b567b73..ea981d7b7 100644 --- a/ide/coq_lex.mll +++ b/ide/coq_lex.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - { open Lexing diff --git a/ide/coq_tactics.ml b/ide/coq_tactics.ml index c6e1f1a44..307ee2522 100644 --- a/ide/coq_tactics.ml +++ b/ide/coq_tactics.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - let tactics = [ "Abstract"; "Absurd"; diff --git a/ide/coq_tactics.mli b/ide/coq_tactics.mli index c31933baa..41219fdf6 100644 --- a/ide/coq_tactics.mli +++ b/ide/coq_tactics.mli @@ -6,7 +6,5 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val tactics : string list diff --git a/ide/coqide.ml b/ide/coqide.ml index 8dc486756..32f2bdd71 100644 --- a/ide/coqide.ml +++ b/ide/coqide.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Preferences open Vernacexpr open Coq diff --git a/ide/coqide.mli b/ide/coqide.mli index 4c01e747a..f91ce0184 100644 --- a/ide/coqide.mli +++ b/ide/coqide.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* The CoqIde main module. The following function [start] will parse the command line, initialize the load path, load the input state, load the files given on the command line, load the ressource file, diff --git a/ide/gtk_parsing.ml b/ide/gtk_parsing.ml index e92a345e3..5411499ca 100644 --- a/ide/gtk_parsing.ml +++ b/ide/gtk_parsing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: coqide.ml 11952 2009-03-02 15:29:08Z vgross $ *) - open Ideutils diff --git a/ide/highlight.mll b/ide/highlight.mll index 3acdd4f08..0a623ca38 100644 --- a/ide/highlight.mll +++ b/ide/highlight.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - { open Lexing diff --git a/ide/ideproof.ml b/ide/ideproof.ml index 700b5a729..3d86f52c6 100644 --- a/ide/ideproof.ml +++ b/ide/ideproof.ml @@ -7,8 +7,6 @@ (************************************************************************) -(* $Id$ *) - (* tag is the tag to be hooked, item is the item covered by this tag, make_menu * * is the template for building menu if needed, sel_cb is the callback if * there diff --git a/ide/ideutils.ml b/ide/ideutils.ml index 14e803899..aaade8aa5 100644 --- a/ide/ideutils.ml +++ b/ide/ideutils.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Preferences diff --git a/ide/ideutils.mli b/ide/ideutils.mli index fbd5af44e..0d57b855e 100644 --- a/ide/ideutils.mli +++ b/ide/ideutils.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val async : ('a -> unit) -> 'a -> unit val sync : ('a -> 'b) -> 'a -> 'b diff --git a/ide/preferences.ml b/ide/preferences.ml index 4e87d1df4..b8eb07cc5 100644 --- a/ide/preferences.ml +++ b/ide/preferences.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Configwin open Printf open Util diff --git a/ide/preferences.mli b/ide/preferences.mli index 6ee7918fe..cd955d7bd 100644 --- a/ide/preferences.mli +++ b/ide/preferences.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - type pref = { mutable cmd_coqc : string; diff --git a/ide/tags.ml b/ide/tags.ml index 842ac53bc..3b407a19d 100644 --- a/ide/tags.ml +++ b/ide/tags.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - let make_tag (tt:GText.tag_table) ~name prop = let new_tag = GText.tag ~name () in diff --git a/ide/typed_notebook.ml b/ide/typed_notebook.ml index cadb5941e..bd26bab27 100644 --- a/ide/typed_notebook.ml +++ b/ide/typed_notebook.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: coqide.ml 11952 2009-03-02 15:29:08Z vgross $ *) - class ['a] typed_notebook default_build nb = object(self) inherit GPack.notebook nb as super diff --git a/ide/undo.ml b/ide/undo.ml index 18c2f7a4d..56b8196bb 100644 --- a/ide/undo.ml +++ b/ide/undo.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open GText open Ideutils type action = diff --git a/ide/undo_lablgtk_ge212.mli b/ide/undo_lablgtk_ge212.mli index 32717fa8e..d7c12de8e 100644 --- a/ide/undo_lablgtk_ge212.mli +++ b/ide/undo_lablgtk_ge212.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: undo_lablgtk_ge26.mli 7580 2005-11-18 17:09:10Z herbelin $ i*) - (* An undoable view class *) class undoable_view : [> Gtk.text_view] Gtk.obj -> diff --git a/ide/undo_lablgtk_ge26.mli b/ide/undo_lablgtk_ge26.mli index 52bd67215..ab51a66b2 100644 --- a/ide/undo_lablgtk_ge26.mli +++ b/ide/undo_lablgtk_ge26.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* An undoable view class *) class undoable_view : [> Gtk.text_view] Gtk.obj -> diff --git a/ide/undo_lablgtk_lt26.mli b/ide/undo_lablgtk_lt26.mli index 46ecfb1d7..330accc7b 100644 --- a/ide/undo_lablgtk_lt26.mli +++ b/ide/undo_lablgtk_lt26.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* An undoable view class *) class undoable_view : Gtk.text_view Gtk.obj -> diff --git a/ide/utf8_convert.mll b/ide/utf8_convert.mll index 82b305347..b1eb0f4c2 100644 --- a/ide/utf8_convert.mll +++ b/ide/utf8_convert.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - { open Lexing let b = Buffer.create 127 diff --git a/ide/utils/config_file.ml b/ide/utils/config_file.ml index 37f2e9a4a..921d3d9c9 100644 --- a/ide/utils/config_file.ml +++ b/ide/utils/config_file.ml @@ -23,8 +23,6 @@ (* *) (*********************************************************************************) -(* $Id$ *) - (* TODO *) (* section comments *) (* better obsoletes: no "{}", line cuts *) diff --git a/interp/constrextern.ml b/interp/constrextern.ml index 99c627a95..fec00c65a 100644 --- a/interp/constrextern.ml +++ b/interp/constrextern.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Pp open Util diff --git a/interp/constrextern.mli b/interp/constrextern.mli index ac9ed5714..ac3a38833 100644 --- a/interp/constrextern.mli +++ b/interp/constrextern.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/interp/constrintern.ml b/interp/constrintern.ml index 2b16023f0..ecaba603d 100644 --- a/interp/constrintern.ml +++ b/interp/constrintern.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Flags diff --git a/interp/constrintern.mli b/interp/constrintern.mli index 4ba2bc587..bf28e0850 100644 --- a/interp/constrintern.mli +++ b/interp/constrintern.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Sign diff --git a/interp/coqlib.ml b/interp/coqlib.ml index 1ca82e35c..6cfe1421f 100644 --- a/interp/coqlib.ml +++ b/interp/coqlib.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/interp/coqlib.mli b/interp/coqlib.mli index 5148461a9..a80e749d3 100644 --- a/interp/coqlib.mli +++ b/interp/coqlib.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Libnames open Nametab diff --git a/interp/dumpglob.ml b/interp/dumpglob.ml index 702c509dc..9dfa808c7 100644 --- a/interp/dumpglob.ml +++ b/interp/dumpglob.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Dump of globalization (to be used by coqdoc) *) diff --git a/interp/dumpglob.mli b/interp/dumpglob.mli index 7235fe172..7efa6f1e0 100644 --- a/interp/dumpglob.mli +++ b/interp/dumpglob.mli @@ -6,9 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: dumpglob.mli 11252 2008-07-24 11:16:48Z notin {% $ %} *) - - val open_glob_file : string -> unit val close_glob_file : unit -> unit diff --git a/interp/genarg.ml b/interp/genarg.ml index 241c92582..e5950cd8d 100644 --- a/interp/genarg.ml +++ b/interp/genarg.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/interp/genarg.mli b/interp/genarg.mli index 50abd351e..984f479fb 100644 --- a/interp/genarg.mli +++ b/interp/genarg.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/interp/implicit_quantifiers.ml b/interp/implicit_quantifiers.ml index d5894b208..89ec5f1f1 100644 --- a/interp/implicit_quantifiers.ml +++ b/interp/implicit_quantifiers.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Decl_kinds diff --git a/interp/implicit_quantifiers.mli b/interp/implicit_quantifiers.mli index 7362d7de5..ac610fe78 100644 --- a/interp/implicit_quantifiers.mli +++ b/interp/implicit_quantifiers.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Decl_kinds open Term diff --git a/interp/modintern.ml b/interp/modintern.ml index 049745ca9..094b723e0 100644 --- a/interp/modintern.ml +++ b/interp/modintern.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/interp/modintern.mli b/interp/modintern.mli index e025447b5..5dacfd070 100644 --- a/interp/modintern.mli +++ b/interp/modintern.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Declarations open Environ open Entries diff --git a/interp/notation.ml b/interp/notation.ml index 794169a37..bfa86b50f 100644 --- a/interp/notation.ml +++ b/interp/notation.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Util open Pp diff --git a/interp/notation.mli b/interp/notation.mli index 91f262b48..224fb1d45 100644 --- a/interp/notation.mli +++ b/interp/notation.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Pp open Bigint diff --git a/interp/ppextend.ml b/interp/ppextend.ml index a4142d694..16d0537b9 100644 --- a/interp/ppextend.ml +++ b/interp/ppextend.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ *) - (*i*) open Pp open Util diff --git a/interp/ppextend.mli b/interp/ppextend.mli index 984696cda..19ca913e8 100644 --- a/interp/ppextend.mli +++ b/interp/ppextend.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names diff --git a/interp/reserve.ml b/interp/reserve.ml index 9d8412825..700fcd1e3 100644 --- a/interp/reserve.ml +++ b/interp/reserve.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Reserved names *) open Util diff --git a/interp/reserve.mli b/interp/reserve.mli index 4cc2eff5a..e53ad8365 100644 --- a/interp/reserve.mli +++ b/interp/reserve.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Rawterm diff --git a/interp/smartlocate.ml b/interp/smartlocate.ml index faad3c50a..424e7cc1e 100644 --- a/interp/smartlocate.ml +++ b/interp/smartlocate.ml @@ -11,8 +11,6 @@ (* This file provides high-level name globalization functions *) -(* $Id:$ *) - (* *) open Pp open Util diff --git a/interp/smartlocate.mli b/interp/smartlocate.mli index b505e7db7..0cd261a82 100644 --- a/interp/smartlocate.mli +++ b/interp/smartlocate.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id:{% $ %} *) - open Util open Names open Libnames diff --git a/interp/syntax_def.ml b/interp/syntax_def.ml index 245ed0f50..334135eaf 100644 --- a/interp/syntax_def.ml +++ b/interp/syntax_def.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/interp/syntax_def.mli b/interp/syntax_def.mli index 6b57b497a..019067608 100644 --- a/interp/syntax_def.mli +++ b/interp/syntax_def.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Topconstr diff --git a/interp/topconstr.ml b/interp/topconstr.ml index c0b624110..5fade008c 100644 --- a/interp/topconstr.ml +++ b/interp/topconstr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Pp open Util diff --git a/interp/topconstr.mli b/interp/topconstr.mli index 02e6d1eeb..2b9506747 100644 --- a/interp/topconstr.mli +++ b/interp/topconstr.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/kernel/byterun/int64_emul.h b/kernel/byterun/int64_emul.h index 04e38656f..86bee72ed 100644 --- a/kernel/byterun/int64_emul.h +++ b/kernel/byterun/int64_emul.h @@ -11,8 +11,6 @@ /* */ /***********************************************************************/ -/* $Id$ */ - /* Software emulation of 64-bit integer arithmetic, for C compilers that do not support it. */ diff --git a/kernel/byterun/int64_native.h b/kernel/byterun/int64_native.h index f5bef4a6f..8a6a26645 100644 --- a/kernel/byterun/int64_native.h +++ b/kernel/byterun/int64_native.h @@ -11,8 +11,6 @@ /* */ /***********************************************************************/ -/* $Id$ */ - /* Wrapper macros around native 64-bit integer arithmetic, so that it has the same interface as the software emulation provided in int64_emul.h */ diff --git a/kernel/closure.ml b/kernel/closure.ml index 93788ed42..e77ea4cb3 100644 --- a/kernel/closure.ml +++ b/kernel/closure.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Term diff --git a/kernel/closure.mli b/kernel/closure.mli index ce339ab33..d482e91b2 100644 --- a/kernel/closure.mli +++ b/kernel/closure.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names open Term diff --git a/kernel/conv_oracle.ml b/kernel/conv_oracle.ml index 0851c7a5f..5e9db9c7d 100644 --- a/kernel/conv_oracle.ml +++ b/kernel/conv_oracle.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Names (* Priority for the expansion of constant in the conversion test. diff --git a/kernel/conv_oracle.mli b/kernel/conv_oracle.mli index 35e09072f..0e8201694 100644 --- a/kernel/conv_oracle.mli +++ b/kernel/conv_oracle.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names (** Order on section paths for unfolding. diff --git a/kernel/cooking.ml b/kernel/cooking.ml index 7605df9eb..7b380944b 100644 --- a/kernel/cooking.ml +++ b/kernel/cooking.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/kernel/cooking.mli b/kernel/cooking.mli index 5f30bce62..42991d507 100644 --- a/kernel/cooking.mli +++ b/kernel/cooking.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/kernel/declarations.ml b/kernel/declarations.ml index 515009798..0762a92d1 100644 --- a/kernel/declarations.ml +++ b/kernel/declarations.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/kernel/declarations.mli b/kernel/declarations.mli index c6cf8a751..15c5350b0 100644 --- a/kernel/declarations.mli +++ b/kernel/declarations.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/kernel/entries.ml b/kernel/entries.ml index 938d1c60a..fb84218cc 100644 --- a/kernel/entries.ml +++ b/kernel/entries.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Univ diff --git a/kernel/entries.mli b/kernel/entries.mli index 2cfdf9314..78316dd9b 100644 --- a/kernel/entries.mli +++ b/kernel/entries.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/kernel/environ.ml b/kernel/environ.ml index 8f6a619a0..69220908e 100644 --- a/kernel/environ.ml +++ b/kernel/environ.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Sign diff --git a/kernel/environ.mli b/kernel/environ.mli index fce149e10..0ecfa21b6 100644 --- a/kernel/environ.mli +++ b/kernel/environ.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/kernel/esubst.ml b/kernel/esubst.ml index c8b5fb269..fd07d9297 100644 --- a/kernel/esubst.ml +++ b/kernel/esubst.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util (*********************) diff --git a/kernel/esubst.mli b/kernel/esubst.mli index bbb3d838e..fd7753093 100644 --- a/kernel/esubst.mli +++ b/kernel/esubst.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Sect } *) (** Explicit substitutions of type ['a]. - ESID(n) = %n END bounded identity diff --git a/kernel/indtypes.ml b/kernel/indtypes.ml index 10cedbf59..90ddd984d 100644 --- a/kernel/indtypes.ml +++ b/kernel/indtypes.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/kernel/indtypes.mli b/kernel/indtypes.mli index c29e5475d..388eb21e4 100644 --- a/kernel/indtypes.mli +++ b/kernel/indtypes.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/kernel/inductive.ml b/kernel/inductive.ml index 76de25344..9215ac0c6 100644 --- a/kernel/inductive.ml +++ b/kernel/inductive.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/kernel/inductive.mli b/kernel/inductive.mli index 7f2b08844..259e1decd 100644 --- a/kernel/inductive.mli +++ b/kernel/inductive.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/kernel/mod_subst.ml b/kernel/mod_subst.ml index 5cb53d166..8abfe0943 100644 --- a/kernel/mod_subst.ml +++ b/kernel/mod_subst.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/kernel/mod_subst.mli b/kernel/mod_subst.mli index 53925955e..e22a3eb7d 100644 --- a/kernel/mod_subst.mli +++ b/kernel/mod_subst.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 [Mod_subst] } *) open Names diff --git a/kernel/mod_typing.ml b/kernel/mod_typing.ml index c9d9ac924..e67b987a6 100644 --- a/kernel/mod_typing.ml +++ b/kernel/mod_typing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Names open Univ diff --git a/kernel/mod_typing.mli b/kernel/mod_typing.mli index 188e4809c..10619820e 100644 --- a/kernel/mod_typing.mli +++ b/kernel/mod_typing.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Declarations open Environ open Entries diff --git a/kernel/modops.ml b/kernel/modops.ml index 2d9c92afc..084fdd4f4 100644 --- a/kernel/modops.ml +++ b/kernel/modops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Pp diff --git a/kernel/modops.mli b/kernel/modops.mli index 0c61e773b..3ab2961d2 100644 --- a/kernel/modops.mli +++ b/kernel/modops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Univ diff --git a/kernel/names.ml b/kernel/names.ml index 06ca87b4d..dfa73e95a 100644 --- a/kernel/names.ml +++ b/kernel/names.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util diff --git a/kernel/names.mli b/kernel/names.mli index f712c8d19..ffbc02714 100644 --- a/kernel/names.mli +++ b/kernel/names.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Identifiers } *) type identifier diff --git a/kernel/pre_env.ml b/kernel/pre_env.ml index b58951e98..3835c81c5 100644 --- a/kernel/pre_env.ml +++ b/kernel/pre_env.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Sign diff --git a/kernel/pre_env.mli b/kernel/pre_env.mli index 619c1afcb..9078558a9 100644 --- a/kernel/pre_env.mli +++ b/kernel/pre_env.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: pre_env.mli 12406 2009-10-21 15:12:52Z soubiran {% $ %} *) - open Util open Names open Sign diff --git a/kernel/reduction.ml b/kernel/reduction.ml index 92386c4d3..4a4661f99 100644 --- a/kernel/reduction.ml +++ b/kernel/reduction.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/kernel/reduction.mli b/kernel/reduction.mli index 06d4478b2..a6ebda491 100644 --- a/kernel/reduction.mli +++ b/kernel/reduction.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Environ open Closure diff --git a/kernel/retroknowledge.ml b/kernel/retroknowledge.ml index a3e493db9..c0f714f96 100644 --- a/kernel/retroknowledge.ml +++ b/kernel/retroknowledge.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Names diff --git a/kernel/retroknowledge.mli b/kernel/retroknowledge.mli index 19f30cd8f..0634a99aa 100644 --- a/kernel/retroknowledge.mli +++ b/kernel/retroknowledge.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term diff --git a/kernel/safe_typing.ml b/kernel/safe_typing.ml index d9c7c9de0..cffe7e772 100644 --- a/kernel/safe_typing.ml +++ b/kernel/safe_typing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/kernel/safe_typing.mli b/kernel/safe_typing.mli index 2aad2eb8c..ce62eeafc 100644 --- a/kernel/safe_typing.mli +++ b/kernel/safe_typing.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/kernel/sign.ml b/kernel/sign.ml index d30d70860..f987a1f6c 100644 --- a/kernel/sign.ml +++ b/kernel/sign.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Names open Util open Term diff --git a/kernel/sign.mli b/kernel/sign.mli index 5cadb125f..07f3df19e 100644 --- a/kernel/sign.mli +++ b/kernel/sign.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term diff --git a/kernel/subtyping.ml b/kernel/subtyping.ml index e07af3ba3..9bc719e7e 100644 --- a/kernel/subtyping.ml +++ b/kernel/subtyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/kernel/subtyping.mli b/kernel/subtyping.mli index d68d908a0..061a6eb0b 100644 --- a/kernel/subtyping.mli +++ b/kernel/subtyping.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Univ open Declarations open Environ diff --git a/kernel/term.ml b/kernel/term.ml index d0e9d1695..a1effb317 100644 --- a/kernel/term.ml +++ b/kernel/term.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This module instantiates the structure of generic deBruijn terms to Coq *) open Util diff --git a/kernel/term.mli b/kernel/term.mli index 830e7e5ed..3940d74c5 100644 --- a/kernel/term.mli +++ b/kernel/term.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names diff --git a/kernel/term_typing.ml b/kernel/term_typing.ml index c465adfac..dac8ee47a 100644 --- a/kernel/term_typing.ml +++ b/kernel/term_typing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/kernel/term_typing.mli b/kernel/term_typing.mli index d1fc71eb5..49463e75a 100644 --- a/kernel/term_typing.mli +++ b/kernel/term_typing.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Univ diff --git a/kernel/type_errors.ml b/kernel/type_errors.ml index 2d26d27e1..77b69bb88 100644 --- a/kernel/type_errors.ml +++ b/kernel/type_errors.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Names open Term open Sign diff --git a/kernel/type_errors.mli b/kernel/type_errors.mli index ed2ec1302..dabff8360 100644 --- a/kernel/type_errors.mli +++ b/kernel/type_errors.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/kernel/typeops.ml b/kernel/typeops.ml index 27db208c6..231ea2b16 100644 --- a/kernel/typeops.ml +++ b/kernel/typeops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/kernel/typeops.mli b/kernel/typeops.mli index a89aae4d2..e2df7e983 100644 --- a/kernel/typeops.mli +++ b/kernel/typeops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/kernel/univ.ml b/kernel/univ.ml index 0a22733d0..f42b6fb93 100644 --- a/kernel/univ.ml +++ b/kernel/univ.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Initial Caml version originates from CoC 4.8 [Dec 1988] *) (* Extension with algebraic universes by HH [Sep 2001] *) (* Additional support for sort-polymorphic inductive types by HH [Mar 2006] *) diff --git a/kernel/univ.mli b/kernel/univ.mli index 1d85386c5..3a2ec557f 100644 --- a/kernel/univ.mli +++ b/kernel/univ.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Universes. *) type universe diff --git a/kernel/vm.ml b/kernel/vm.ml index 338936250..1f57457d7 100644 --- a/kernel/vm.ml +++ b/kernel/vm.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Names open Term open Conv_oracle diff --git a/lib/bigint.ml b/lib/bigint.ml index f505bbe14..a3462faa1 100644 --- a/lib/bigint.ml +++ b/lib/bigint.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Pp (*i*) diff --git a/lib/bigint.mli b/lib/bigint.mli index 06f542227..348c6c5d9 100644 --- a/lib/bigint.mli +++ b/lib/bigint.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp (** Arbitrary large integer numbers *) diff --git a/lib/dnet.ml b/lib/dnet.ml index f7b369297..a0c301145 100644 --- a/lib/dnet.ml +++ b/lib/dnet.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id:$ *) - (* Generic dnet implementation over non-recursive types *) module type Datatype = diff --git a/lib/dnet.mli b/lib/dnet.mli index 8b50fae23..be33ecc6a 100644 --- a/lib/dnet.mli +++ b/lib/dnet.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id:{% $ %} *) - (** Generic discrimination net implementation over recursive types. This module implements a association data structure similar to tries but working on any types (not just lists). It is a term diff --git a/lib/dyn.ml b/lib/dyn.ml index d2bd458a7..a2548fa69 100644 --- a/lib/dyn.ml +++ b/lib/dyn.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util (* Dynamics, programmed with DANGER !!! *) diff --git a/lib/dyn.mli b/lib/dyn.mli index befc8de7e..235dae3af 100644 --- a/lib/dyn.mli +++ b/lib/dyn.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Dynamics. Use with extreme care. Not for kids. *) type t diff --git a/lib/explore.ml b/lib/explore.ml index 760495099..b227112b2 100644 --- a/lib/explore.ml +++ b/lib/explore.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Format (*s Definition of a search problem. *) diff --git a/lib/explore.mli b/lib/explore.mli index 34a472b72..0e8eb32be 100644 --- a/lib/explore.mli +++ b/lib/explore.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Search strategies. } *) (** {6 Sect } *) diff --git a/lib/flags.ml b/lib/flags.ml index 555739b11..cb87e2f2b 100644 --- a/lib/flags.ml +++ b/lib/flags.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - let with_option o f x = let old = !o in o:=true; try let r = f x in o := old; r diff --git a/lib/flags.mli b/lib/flags.mli index 404cc2d85..8576a7e5e 100644 --- a/lib/flags.mli +++ b/lib/flags.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Global options of the system. *) val boot : bool ref diff --git a/lib/gmap.ml b/lib/gmap.ml index 0c498fe7d..fc9965258 100644 --- a/lib/gmap.ml +++ b/lib/gmap.ml @@ -5,7 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) (* Maps using the generic comparison function of ocaml. Code borrowed from the ocaml standard library (Copyright 1996, INRIA). *) diff --git a/lib/gmap.mli b/lib/gmap.mli index 7c86120c6..45b04151e 100644 --- a/lib/gmap.mli +++ b/lib/gmap.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Maps using the generic comparison function of ocaml. Same interface as the module [Map] from the ocaml standard library. *) diff --git a/lib/gmapl.ml b/lib/gmapl.ml index cec10d644..ef8a04f28 100644 --- a/lib/gmapl.ml +++ b/lib/gmapl.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util type ('a,'b) t = ('a,'b list) Gmap.t diff --git a/lib/gmapl.mli b/lib/gmapl.mli index 349774073..fdc42e3ad 100644 --- a/lib/gmapl.mli +++ b/lib/gmapl.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Maps from ['a] to lists of ['b]. *) type ('a,'b) t diff --git a/lib/gset.ml b/lib/gset.ml index d39cb23f2..7439e822d 100644 --- a/lib/gset.ml +++ b/lib/gset.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Sets using the generic comparison function of ocaml. Code borrowed from the ocaml standard library. *) diff --git a/lib/gset.mli b/lib/gset.mli index 0b80176d5..265f8eb34 100644 --- a/lib/gset.mli +++ b/lib/gset.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Sets using the generic comparison function of ocaml. Same interface as the module [Set] from the ocaml standard library. *) diff --git a/lib/hashcons.ml b/lib/hashcons.ml index 921a4ed56..5e6f31179 100644 --- a/lib/hashcons.ml +++ b/lib/hashcons.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Hash consing of datastructures *) (* The generic hash-consing functions (does not use Obj) *) diff --git a/lib/hashcons.mli b/lib/hashcons.mli index ca66730b2..2b3b7dfb0 100644 --- a/lib/hashcons.mli +++ b/lib/hashcons.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Generic hash-consing. *) module type Comp = diff --git a/lib/heap.ml b/lib/heap.ml index 7ddb4a720..f1878f2ab 100644 --- a/lib/heap.ml +++ b/lib/heap.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*s Heaps *) module type Ordered = sig diff --git a/lib/heap.mli b/lib/heap.mli index a8c70d37d..fe34b250d 100644 --- a/lib/heap.mli +++ b/lib/heap.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Heaps *) module type Ordered = sig diff --git a/lib/option.ml b/lib/option.ml index 942fff48a..cd145d1c3 100644 --- a/lib/option.ml +++ b/lib/option.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Module implementing basic combinators for OCaml option type. It tries follow closely the style of OCaml standard library. diff --git a/lib/option.mli b/lib/option.mli index 3711a2efd..b37d905f5 100644 --- a/lib/option.mli +++ b/lib/option.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: option.mli 12603 2009-12-21 11:16:27Z herbelin {% $ %} *) - (** Module implementing basic combinators for OCaml option type. It tries follow closely the style of OCaml standard library. diff --git a/lib/pp.ml4 b/lib/pp.ml4 index b0948b0f4..405919673 100644 --- a/lib/pp.ml4 +++ b/lib/pp.ml4 @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp_control (* This should not be used outside of this file. Use diff --git a/lib/pp.mli b/lib/pp.mli index 6ddfa6fc9..56e66225c 100644 --- a/lib/pp.mli +++ b/lib/pp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp_control (** Modify pretty printing functions behavior for emacs ouput (special diff --git a/lib/pp_control.ml b/lib/pp_control.ml index ecc546491..cd92cc352 100644 --- a/lib/pp_control.ml +++ b/lib/pp_control.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Parameters of pretty-printing *) type pp_global_params = { diff --git a/lib/pp_control.mli b/lib/pp_control.mli index 83ee7a0f3..fe1ee6de3 100644 --- a/lib/pp_control.mli +++ b/lib/pp_control.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Parameters of pretty-printing. *) type pp_global_params = { diff --git a/lib/predicate.ml b/lib/predicate.ml index af66c0f28..e419aa6e9 100644 --- a/lib/predicate.ml +++ b/lib/predicate.ml @@ -10,8 +10,6 @@ (* *) (************************************************************************) -(* $Id$ *) - (* Sets over ordered types *) module type OrderedType = diff --git a/lib/predicate.mli b/lib/predicate.mli index 862479ec4..bcc89e727 100644 --- a/lib/predicate.mli +++ b/lib/predicate.mli @@ -1,6 +1,4 @@ -(*i $Id$ i*) - (** Module [Pred]: sets over infinite ordered types with complement. *) (** This module implements the set data structure, given a total ordering diff --git a/lib/profile.ml b/lib/profile.ml index 78caf0148..d15447817 100644 --- a/lib/profile.ml +++ b/lib/profile.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Gc let word_length = Sys.word_size / 8 diff --git a/lib/profile.mli b/lib/profile.mli index 3d64b79c1..1934b0482 100644 --- a/lib/profile.mli +++ b/lib/profile.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 This program is a small time and allocation profiler for Objective Caml } *) (*i It requires the UNIX library *) diff --git a/lib/rtree.ml b/lib/rtree.ml index ad4d31338..b1c934506 100644 --- a/lib/rtree.ml +++ b/lib/rtree.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util diff --git a/lib/rtree.mli b/lib/rtree.mli index 6dd66d104..42723358d 100644 --- a/lib/rtree.mli +++ b/lib/rtree.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Type of regular tree with nodes labelled by values of type 'a The implementation uses de Bruijn indices, so binding capture is avoided by the lift operator (see example below) *) diff --git a/lib/safe_marshal.ml b/lib/safe_marshal.ml index 88101b5d2..e9ba81b49 100644 --- a/lib/safe_marshal.ml +++ b/lib/safe_marshal.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - let hobcnv = Array.init 256 (fun i -> Printf.sprintf "%.2x" i) let bohcnv = Array.init 256 (fun i -> i - (if 0x30 <= i then 0x30 else 0) - diff --git a/lib/store.ml b/lib/store.ml index 8f1309531..bc1b335fd 100644 --- a/lib/store.ml +++ b/lib/store.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (*** This module implements an "untyped store", in this particular case we see it as an extensible record whose fields are left unspecified. ***) diff --git a/lib/store.mli b/lib/store.mli index 0caeb2abb..5df0c99a7 100644 --- a/lib/store.mli +++ b/lib/store.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (*** This module implements an "untyped store", in this particular case we see it as an extensible record whose fields are left unspecified. ***) diff --git a/lib/system.ml b/lib/system.ml index 4b657e485..2391b99e0 100644 --- a/lib/system.ml +++ b/lib/system.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Unix diff --git a/lib/system.mli b/lib/system.mli index 8eb375804..09142f365 100644 --- a/lib/system.mli +++ b/lib/system.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Sect } *) (** Files and load paths. Load path entries remember the original root given by the user. For efficiency, we keep the full path (field diff --git a/lib/tlm.ml b/lib/tlm.ml index 1c1483ad4..a3d4d1a03 100644 --- a/lib/tlm.ml +++ b/lib/tlm.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - type ('a,'b) t = Node of 'b Gset.t * ('a, ('a,'b) t) Gmap.t let empty = Node (Gset.empty, Gmap.empty) diff --git a/lib/tlm.mli b/lib/tlm.mli index 05ecee871..e4c980696 100644 --- a/lib/tlm.mli +++ b/lib/tlm.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Tries. This module implements a data structure [('a,'b) t] mapping lists of values of type ['a] to sets (as lists) of values of type ['b]. *) diff --git a/lib/util.ml b/lib/util.ml index ce98d3234..a70278d57 100644 --- a/lib/util.ml +++ b/lib/util.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - open Pp (* Errors *) diff --git a/lib/util.mli b/lib/util.mli index ecf6b0a16..fd8ff9275 100644 --- a/lib/util.mli +++ b/lib/util.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 **********************************************************************) -(*i $Id$ i*) - open Pp (** This module contains numerous utility functions on strings, lists, diff --git a/library/decl_kinds.ml b/library/decl_kinds.ml index 5fd27f467..be2e79c70 100644 --- a/library/decl_kinds.ml +++ b/library/decl_kinds.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Libnames diff --git a/library/decl_kinds.mli b/library/decl_kinds.mli index abc201eb1..2c04d0fdd 100644 --- a/library/decl_kinds.mli +++ b/library/decl_kinds.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: decl_kinds.mli 12337 2009-09-17 15:58:14Z glondu {% $ %} *) - open Util open Libnames diff --git a/library/declare.ml b/library/declare.ml index a83a7b4b0..68b9ca9fb 100644 --- a/library/declare.ml +++ b/library/declare.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** This module is about the low-level declaration of logical objects *) open Pp diff --git a/library/declare.mli b/library/declare.mli index 1b4564d9c..db9e1aa6d 100644 --- a/library/declare.mli +++ b/library/declare.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Libnames open Term diff --git a/library/declaremods.ml b/library/declaremods.ml index bca52c556..42abebe86 100644 --- a/library/declaremods.ml +++ b/library/declaremods.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/library/declaremods.mli b/library/declaremods.mli index 17fd44024..4cbdf4ce4 100644 --- a/library/declaremods.mli +++ b/library/declaremods.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Entries diff --git a/library/decls.ml b/library/decls.ml index ac2203ccf..7243eb0f6 100644 --- a/library/decls.ml +++ b/library/decls.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** This module registers tables for some non-logical informations associated declarations *) diff --git a/library/decls.mli b/library/decls.mli index 091ec7d99..34a96cd8b 100644 --- a/library/decls.mli +++ b/library/decls.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Sign open Libnames diff --git a/library/dischargedhypsmap.ml b/library/dischargedhypsmap.ml index 85de6ab8f..0154f4334 100644 --- a/library/dischargedhypsmap.ml +++ b/library/dischargedhypsmap.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Libnames open Names diff --git a/library/dischargedhypsmap.mli b/library/dischargedhypsmap.mli index bc9541cf4..b264c1228 100644 --- a/library/dischargedhypsmap.mli +++ b/library/dischargedhypsmap.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Libnames open Term open Environ diff --git a/library/global.ml b/library/global.ml index d5fafbb8b..a7cd61184 100644 --- a/library/global.ml +++ b/library/global.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/library/global.mli b/library/global.mli index 17ad57138..ae2ed16f7 100644 --- a/library/global.mli +++ b/library/global.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Univ open Term diff --git a/library/goptions.ml b/library/goptions.ml index 06d4b618e..e23bee15d 100644 --- a/library/goptions.ml +++ b/library/goptions.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This module manages customization parameters at the vernacular level *) open Pp diff --git a/library/goptions.mli b/library/goptions.mli index a8ed8a045..c63845ae0 100644 --- a/library/goptions.mli +++ b/library/goptions.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** This module manages customization parameters at the vernacular level *) (** Two kinds of things are managed : tables and options value diff --git a/library/heads.ml b/library/heads.ml index 056f78a5f..1f2cdc6f9 100644 --- a/library/heads.ml +++ b/library/heads.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/library/heads.mli b/library/heads.mli index bddee835f..5a0df8423 100644 --- a/library/heads.mli +++ b/library/heads.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: heads.mli 10841 2008-04-24 07:19:57Z herbelin {% $ %} *) - open Names open Term open Environ diff --git a/library/impargs.ml b/library/impargs.ml index b53b2a89d..f7d998d8c 100644 --- a/library/impargs.ml +++ b/library/impargs.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Libnames diff --git a/library/impargs.mli b/library/impargs.mli index dc66e5493..f43880e29 100644 --- a/library/impargs.mli +++ b/library/impargs.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Libnames open Term diff --git a/library/lib.ml b/library/lib.ml index c8f5c6258..dcf7e70cd 100644 --- a/library/lib.ml +++ b/library/lib.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Libnames diff --git a/library/lib.mli b/library/lib.mli index e8b905f26..f1e64e69a 100644 --- a/library/lib.mli +++ b/library/lib.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Sect } *) (** This module provides a general mechanism to keep a trace of all operations diff --git a/library/libnames.ml b/library/libnames.ml index 9a7135eae..13f678c5e 100644 --- a/library/libnames.ml +++ b/library/libnames.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/library/libnames.mli b/library/libnames.mli index 9da6a0d5c..9db6d787d 100644 --- a/library/libnames.mli +++ b/library/libnames.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/library/libobject.ml b/library/libobject.ml index ecdcacf1d..8577ae333 100644 --- a/library/libobject.ml +++ b/library/libobject.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Libnames diff --git a/library/libobject.mli b/library/libobject.mli index 8b21971aa..5a48419c9 100644 --- a/library/libobject.mli +++ b/library/libobject.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Libnames open Mod_subst diff --git a/library/library.ml b/library/library.ml index fbe437fc4..8677de837 100644 --- a/library/library.ml +++ b/library/library.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util diff --git a/library/library.mli b/library/library.mli index 05b213350..9bbb45143 100644 --- a/library/library.mli +++ b/library/library.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Libnames diff --git a/library/nameops.ml b/library/nameops.ml index 28b799f53..0a0fce42b 100644 --- a/library/nameops.ml +++ b/library/nameops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/library/nameops.mli b/library/nameops.mli index 414ee94ad..0f1d52420 100644 --- a/library/nameops.mli +++ b/library/nameops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names (** Identifiers and names *) diff --git a/library/nametab.ml b/library/nametab.ml index c14b6cfc0..4bb9f104d 100644 --- a/library/nametab.ml +++ b/library/nametab.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/library/nametab.mli b/library/nametab.mli index 749d00343..a464fd9a9 100755 --- a/library/nametab.mli +++ b/library/nametab.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Pp open Names diff --git a/library/states.ml b/library/states.ml index c4e766095..ed13c3b7a 100644 --- a/library/states.ml +++ b/library/states.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open System type state = Lib.frozen * Summary.frozen diff --git a/library/states.mli b/library/states.mli index fb11756e5..f0dab29f2 100644 --- a/library/states.mli +++ b/library/states.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Sect } *) (** States of the system. In that module, we provide functions to get and set the state of the whole system. Internally, it is done by diff --git a/library/summary.ml b/library/summary.ml index e9b0bbd36..b9c07ac85 100644 --- a/library/summary.ml +++ b/library/summary.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util diff --git a/library/summary.mli b/library/summary.mli index 58272aadb..0f6aaddaf 100644 --- a/library/summary.mli +++ b/library/summary.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** This module registers the declaration of global tables, which will be kept in synchronization during the various backtracks of the system. *) diff --git a/parsing/argextend.ml4 b/parsing/argextend.ml4 index 89edbb123..3b2160af1 100644 --- a/parsing/argextend.ml4 +++ b/parsing/argextend.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo q_MLast.cmo" i*) -(* $Id$ *) - open Genarg open Q_util open Q_coqast diff --git a/parsing/egrammar.ml b/parsing/egrammar.ml index b5ee1ae60..337ddd7ed 100644 --- a/parsing/egrammar.ml +++ b/parsing/egrammar.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Pcoq diff --git a/parsing/egrammar.mli b/parsing/egrammar.mli index 50132fd38..1e9159933 100644 --- a/parsing/egrammar.mli +++ b/parsing/egrammar.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Topconstr diff --git a/parsing/extend.ml b/parsing/extend.ml index 7643120f3..a3ef4893a 100644 --- a/parsing/extend.ml +++ b/parsing/extend.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util (**********************************************************************) diff --git a/parsing/extend.mli b/parsing/extend.mli index 6bf8165eb..5ff475f79 100644 --- a/parsing/extend.mli +++ b/parsing/extend.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util (********************************************************************* diff --git a/parsing/extrawit.ml b/parsing/extrawit.ml index 122730f72..7ccff5435 100644 --- a/parsing/extrawit.ml +++ b/parsing/extrawit.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Genarg diff --git a/parsing/extrawit.mli b/parsing/extrawit.mli index f15c388b6..b330a8e64 100644 --- a/parsing/extrawit.mli +++ b/parsing/extrawit.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Genarg open Tacexpr diff --git a/parsing/g_constr.ml4 b/parsing/g_constr.ml4 index 393125e29..432903377 100644 --- a/parsing/g_constr.ml4 +++ b/parsing/g_constr.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pp open Pcoq open Constr diff --git a/parsing/g_ltac.ml4 b/parsing/g_ltac.ml4 index 0e97b2a7f..ca9e90cd5 100644 --- a/parsing/g_ltac.ml4 +++ b/parsing/g_ltac.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pp open Util open Topconstr diff --git a/parsing/g_natsyntax.mli b/parsing/g_natsyntax.mli index 20f5c1bfd..3751f603b 100644 --- a/parsing/g_natsyntax.mli +++ b/parsing/g_natsyntax.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Nice syntax for naturals. *) open Notation diff --git a/parsing/g_prim.ml4 b/parsing/g_prim.ml4 index 6e7acd3f5..02b3df3fb 100644 --- a/parsing/g_prim.ml4 +++ b/parsing/g_prim.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(*i $Id$ i*) - open Pcoq open Names open Libnames diff --git a/parsing/g_proofs.ml4 b/parsing/g_proofs.ml4 index 27ad1e964..758d4599a 100644 --- a/parsing/g_proofs.ml4 +++ b/parsing/g_proofs.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pcoq open Pp diff --git a/parsing/g_tactic.ml4 b/parsing/g_tactic.ml4 index c845daf2c..0ef18de2f 100644 --- a/parsing/g_tactic.ml4 +++ b/parsing/g_tactic.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pp open Pcoq open Util diff --git a/parsing/g_vernac.ml4 b/parsing/g_vernac.ml4 index db683b9a9..29b51322d 100644 --- a/parsing/g_vernac.ml4 +++ b/parsing/g_vernac.ml4 @@ -9,8 +9,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pp open Util diff --git a/parsing/g_xml.ml4 b/parsing/g_xml.ml4 index 0f7029041..8bda1e58f 100644 --- a/parsing/g_xml.ml4 +++ b/parsing/g_xml.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo" i*) -(* $Id$ *) - open Pp open Util open Names diff --git a/parsing/g_zsyntax.mli b/parsing/g_zsyntax.mli index c4f39f80b..29dd60f35 100644 --- a/parsing/g_zsyntax.mli +++ b/parsing/g_zsyntax.mli @@ -6,6 +6,4 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Nice syntax for integers. *) diff --git a/parsing/lexer.ml4 b/parsing/lexer.ml4 index 4b15e200c..afb26ec81 100644 --- a/parsing/lexer.ml4 +++ b/parsing/lexer.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_macro.cmo" i*) -(*i $Id$ i*) - open Pp open Util open Token diff --git a/parsing/lexer.mli b/parsing/lexer.mli index aabac79fb..09492ceb1 100644 --- a/parsing/lexer.mli +++ b/parsing/lexer.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util diff --git a/parsing/pcoq.ml4 b/parsing/pcoq.ml4 index de15d8a7c..e11cdd96f 100644 --- a/parsing/pcoq.ml4 +++ b/parsing/pcoq.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo pa_macro.cmo" i*) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/parsing/pcoq.mli b/parsing/pcoq.mli index f9e65acac..23d85d94a 100644 --- a/parsing/pcoq.mli +++ b/parsing/pcoq.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Rawterm diff --git a/parsing/ppconstr.ml b/parsing/ppconstr.ml index 08ac7fd68..597505686 100644 --- a/parsing/ppconstr.ml +++ b/parsing/ppconstr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Util open Pp diff --git a/parsing/ppconstr.mli b/parsing/ppconstr.mli index d2d44f245..2becdbcfd 100644 --- a/parsing/ppconstr.mli +++ b/parsing/ppconstr.mli @@ -7,8 +7,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Environ open Term diff --git a/parsing/pptactic.ml b/parsing/pptactic.ml index 5f02daf4a..9714b7fa9 100644 --- a/parsing/pptactic.ml +++ b/parsing/pptactic.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Names open Namegen diff --git a/parsing/pptactic.mli b/parsing/pptactic.mli index a6eacd53a..34a7089fe 100644 --- a/parsing/pptactic.mli +++ b/parsing/pptactic.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Genarg open Tacexpr diff --git a/parsing/ppvernac.ml b/parsing/ppvernac.ml index 470f937c0..99039e867 100644 --- a/parsing/ppvernac.ml +++ b/parsing/ppvernac.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Names open Nameops diff --git a/parsing/ppvernac.mli b/parsing/ppvernac.mli index 6c2916f41..98511f3e5 100644 --- a/parsing/ppvernac.mli +++ b/parsing/ppvernac.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Genarg open Vernacexpr diff --git a/parsing/prettyp.ml b/parsing/prettyp.ml index 98c93f897..882a94ffb 100644 --- a/parsing/prettyp.ml +++ b/parsing/prettyp.ml @@ -10,8 +10,6 @@ * on May-June 2006 for implementation of abstraction of pretty-printing of objects. *) -(* $Id$ *) - open Pp open Util open Names diff --git a/parsing/prettyp.mli b/parsing/prettyp.mli index 04aad9ab4..913ab8b43 100644 --- a/parsing/prettyp.mli +++ b/parsing/prettyp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/parsing/printer.ml b/parsing/printer.ml index cd07c4e15..d3c4ae63d 100644 --- a/parsing/printer.ml +++ b/parsing/printer.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/parsing/printer.mli b/parsing/printer.mli index 6289fa66a..5cd402e9f 100644 --- a/parsing/printer.mli +++ b/parsing/printer.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names open Libnames diff --git a/parsing/q_constr.ml4 b/parsing/q_constr.ml4 index 093910b4d..28911794f 100644 --- a/parsing/q_constr.ml4 +++ b/parsing/q_constr.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo q_MLast.cmo" i*) -(* $Id$ *) - open Rawterm open Term open Names diff --git a/parsing/q_coqast.ml4 b/parsing/q_coqast.ml4 index 1bd5af533..89a1c2ed5 100644 --- a/parsing/q_coqast.ml4 +++ b/parsing/q_coqast.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "q_MLast.cmo pa_macro.cmo" i*) -(* $Id$ *) - open Util open Names open Libnames diff --git a/parsing/q_util.ml4 b/parsing/q_util.ml4 index 7b9037d92..e5851f81d 100644 --- a/parsing/q_util.ml4 +++ b/parsing/q_util.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "q_MLast.cmo" i*) -(* $Id$ *) - (* This file defines standard combinators to build ml expressions *) open Util diff --git a/parsing/q_util.mli b/parsing/q_util.mli index 4fe853702..59b3f334c 100644 --- a/parsing/q_util.mli +++ b/parsing/q_util.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - val patt_of_expr : MLast.expr -> MLast.patt val mlexpr_of_list : ('a -> MLast.expr) -> 'a list -> MLast.expr diff --git a/parsing/tacextend.ml4 b/parsing/tacextend.ml4 index 517e34aa2..f77b24eff 100644 --- a/parsing/tacextend.ml4 +++ b/parsing/tacextend.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo q_MLast.cmo" i*) -(* $Id$ *) - open Util open Genarg open Q_util diff --git a/parsing/tactic_printer.ml b/parsing/tactic_printer.ml index bf554acf6..57af21852 100644 --- a/parsing/tactic_printer.ml +++ b/parsing/tactic_printer.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Sign diff --git a/parsing/tactic_printer.mli b/parsing/tactic_printer.mli index 836c4712b..129f0e671 100644 --- a/parsing/tactic_printer.mli +++ b/parsing/tactic_printer.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Sign open Evd diff --git a/parsing/vernacextend.ml4 b/parsing/vernacextend.ml4 index e1997b878..ff354d5e0 100644 --- a/parsing/vernacextend.ml4 +++ b/parsing/vernacextend.ml4 @@ -8,8 +8,6 @@ (*i camlp4use: "pa_extend.cmo q_MLast.cmo" i*) -(* $Id$ *) - open Util open Genarg open Q_util diff --git a/plugins/cc/ccalgo.ml b/plugins/cc/ccalgo.ml index 9b5fca4da..847b3f610 100644 --- a/plugins/cc/ccalgo.ml +++ b/plugins/cc/ccalgo.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This file implements the basic congruence-closure algorithm by *) (* Downey,Sethi and Tarjan. *) diff --git a/plugins/cc/ccalgo.mli b/plugins/cc/ccalgo.mli index 5f56c7e69..844bd43b5 100644 --- a/plugins/cc/ccalgo.mli +++ b/plugins/cc/ccalgo.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Term open Names diff --git a/plugins/cc/ccproof.ml b/plugins/cc/ccproof.ml index 2a019ebff..e45e4e70a 100644 --- a/plugins/cc/ccproof.ml +++ b/plugins/cc/ccproof.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This file uses the (non-compressed) union-find structure to generate *) (* proof-trees that will be transformed into proof-terms in cctac.ml4 *) diff --git a/plugins/cc/ccproof.mli b/plugins/cc/ccproof.mli index 2a0ca688c..6980ed8c6 100644 --- a/plugins/cc/ccproof.mli +++ b/plugins/cc/ccproof.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Ccalgo open Names open Term diff --git a/plugins/cc/cctac.ml b/plugins/cc/cctac.ml index ccfa2a0a7..1ea1fdc64 100644 --- a/plugins/cc/cctac.ml +++ b/plugins/cc/cctac.ml @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - (* This file is the interface between the c-c algorithm and Coq *) open Evd diff --git a/plugins/cc/cctac.mli b/plugins/cc/cctac.mli index 7ed077bda..00ceac992 100644 --- a/plugins/cc/cctac.mli +++ b/plugins/cc/cctac.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Proof_type diff --git a/plugins/cc/g_congruence.ml4 b/plugins/cc/g_congruence.ml4 index d9db927a3..d65e339a3 100644 --- a/plugins/cc/g_congruence.ml4 +++ b/plugins/cc/g_congruence.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Cctac open Tactics open Tacticals diff --git a/plugins/decl_mode/decl_expr.mli b/plugins/decl_mode/decl_expr.mli index 20a95dabf..b267fdc97 100644 --- a/plugins/decl_mode/decl_expr.mli +++ b/plugins/decl_mode/decl_expr.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id:$ *) - open Names open Util open Tacexpr diff --git a/plugins/decl_mode/decl_interp.ml b/plugins/decl_mode/decl_interp.ml index 2b583af40..1b91ef177 100644 --- a/plugins/decl_mode/decl_interp.ml +++ b/plugins/decl_mode/decl_interp.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Names open Topconstr diff --git a/plugins/decl_mode/decl_interp.mli b/plugins/decl_mode/decl_interp.mli index bd0859382..bb008eaf8 100644 --- a/plugins/decl_mode/decl_interp.mli +++ b/plugins/decl_mode/decl_interp.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Tacinterp open Decl_expr open Mod_subst diff --git a/plugins/decl_mode/decl_mode.ml b/plugins/decl_mode/decl_mode.ml index 90b0085ff..d71e356c7 100644 --- a/plugins/decl_mode/decl_mode.ml +++ b/plugins/decl_mode/decl_mode.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id:$ i*) - open Names open Term open Evd diff --git a/plugins/decl_mode/decl_mode.mli b/plugins/decl_mode/decl_mode.mli index fe485ce9b..0c24cd815 100644 --- a/plugins/decl_mode/decl_mode.mli +++ b/plugins/decl_mode/decl_mode.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id:$ *) - open Names open Term open Evd diff --git a/plugins/decl_mode/decl_proof_instr.ml b/plugins/decl_mode/decl_proof_instr.ml index cd695f239..97a56cabe 100644 --- a/plugins/decl_mode/decl_proof_instr.ml +++ b/plugins/decl_mode/decl_proof_instr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Evd diff --git a/plugins/decl_mode/decl_proof_instr.mli b/plugins/decl_mode/decl_proof_instr.mli index 0b22b7ac5..82df643d1 100644 --- a/plugins/decl_mode/decl_proof_instr.mli +++ b/plugins/decl_mode/decl_proof_instr.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Refiner open Names open Term diff --git a/plugins/decl_mode/g_decl_mode.ml4 b/plugins/decl_mode/g_decl_mode.ml4 index cdfc57b37..d87708510 100644 --- a/plugins/decl_mode/g_decl_mode.ml4 +++ b/plugins/decl_mode/g_decl_mode.ml4 @@ -9,8 +9,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) (*i camlp4use: "pa_extend.cmo q_MLast.cmo" i*) -(* $Id$ *) - (* arnaud: veiller à l'aspect tutorial des commentaires *) open Pp diff --git a/plugins/decl_mode/ppdecl_proof.ml b/plugins/decl_mode/ppdecl_proof.ml index 40c712cdf..5bd15b93f 100644 --- a/plugins/decl_mode/ppdecl_proof.ml +++ b/plugins/decl_mode/ppdecl_proof.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Decl_expr diff --git a/plugins/dp/Dp.v b/plugins/dp/Dp.v index bc7d73f62..1b66c334e 100644 --- a/plugins/dp/Dp.v +++ b/plugins/dp/Dp.v @@ -6,8 +6,6 @@ Require Export Classical. (* Zenon *) (* Copyright 2004 INRIA *) -(* $Id$ *) - Lemma zenon_nottrue : (~True -> False). Proof. tauto. Qed. diff --git a/plugins/dp/g_dp.ml4 b/plugins/dp/g_dp.ml4 index 82f86cd81..e2cd4b3e3 100644 --- a/plugins/dp/g_dp.ml4 +++ b/plugins/dp/g_dp.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Dp TACTIC EXTEND Simplify diff --git a/plugins/dp/zenon.v b/plugins/dp/zenon.v index 502465c6b..89028c4f4 100644 --- a/plugins/dp/zenon.v +++ b/plugins/dp/zenon.v @@ -1,6 +1,4 @@ (* Copyright 2004 INRIA *) -(* $Id$ *) - Require Export Classical. Lemma zenon_nottrue : diff --git a/plugins/extraction/common.ml b/plugins/extraction/common.ml index 73b51cfe7..18b3642e2 100644 --- a/plugins/extraction/common.ml +++ b/plugins/extraction/common.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/plugins/extraction/common.mli b/plugins/extraction/common.mli index a68e72d26..6d33bd8ea 100644 --- a/plugins/extraction/common.mli +++ b/plugins/extraction/common.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Libnames open Miniml diff --git a/plugins/extraction/extract_env.ml b/plugins/extraction/extract_env.ml index 37721c9b9..33bac0e1c 100644 --- a/plugins/extraction/extract_env.ml +++ b/plugins/extraction/extract_env.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Term open Declarations open Names diff --git a/plugins/extraction/extract_env.mli b/plugins/extraction/extract_env.mli index dcb4601e5..243fe4db3 100644 --- a/plugins/extraction/extract_env.mli +++ b/plugins/extraction/extract_env.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s This module declares the extraction commands. *) open Names diff --git a/plugins/extraction/extraction.ml b/plugins/extraction/extraction.ml index e7c2e23f7..e7b5f31fc 100644 --- a/plugins/extraction/extraction.ml +++ b/plugins/extraction/extraction.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/plugins/extraction/extraction.mli b/plugins/extraction/extraction.mli index 6bcd24763..7920a0302 100644 --- a/plugins/extraction/extraction.mli +++ b/plugins/extraction/extraction.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Extraction from Coq terms to Miniml. *) open Names diff --git a/plugins/extraction/haskell.ml b/plugins/extraction/haskell.ml index 579f42df5..84202d539 100644 --- a/plugins/extraction/haskell.ml +++ b/plugins/extraction/haskell.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Production of Haskell syntax. *) open Pp diff --git a/plugins/extraction/haskell.mli b/plugins/extraction/haskell.mli index 1b5dbc711..0a865bfcf 100644 --- a/plugins/extraction/haskell.mli +++ b/plugins/extraction/haskell.mli @@ -6,7 +6,5 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val haskell_descr : Miniml.language_descr diff --git a/plugins/extraction/miniml.mli b/plugins/extraction/miniml.mli index 00df1a98d..effc7af46 100644 --- a/plugins/extraction/miniml.mli +++ b/plugins/extraction/miniml.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Target language for extraction: a core ML called MiniML. *) open Pp diff --git a/plugins/extraction/mlutil.ml b/plugins/extraction/mlutil.ml index df962773d..630a59e9d 100644 --- a/plugins/extraction/mlutil.ml +++ b/plugins/extraction/mlutil.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Pp open Util diff --git a/plugins/extraction/mlutil.mli b/plugins/extraction/mlutil.mli index 0366c4ba7..8691d0181 100644 --- a/plugins/extraction/mlutil.mli +++ b/plugins/extraction/mlutil.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/plugins/extraction/modutil.ml b/plugins/extraction/modutil.ml index 9195b747e..7e8127fb3 100644 --- a/plugins/extraction/modutil.ml +++ b/plugins/extraction/modutil.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Declarations open Environ diff --git a/plugins/extraction/modutil.mli b/plugins/extraction/modutil.mli index 8e04a368e..70d14fb27 100644 --- a/plugins/extraction/modutil.mli +++ b/plugins/extraction/modutil.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Declarations open Environ diff --git a/plugins/extraction/ocaml.ml b/plugins/extraction/ocaml.ml index 5759cf0c2..3d980e65f 100644 --- a/plugins/extraction/ocaml.ml +++ b/plugins/extraction/ocaml.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Production of Ocaml syntax. *) open Pp diff --git a/plugins/extraction/ocaml.mli b/plugins/extraction/ocaml.mli index 4a1c1778f..78cf59740 100644 --- a/plugins/extraction/ocaml.mli +++ b/plugins/extraction/ocaml.mli @@ -6,7 +6,5 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val ocaml_descr : Miniml.language_descr diff --git a/plugins/extraction/scheme.ml b/plugins/extraction/scheme.ml index 9cc34634a..6a44812da 100644 --- a/plugins/extraction/scheme.ml +++ b/plugins/extraction/scheme.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Production of Scheme syntax. *) open Pp diff --git a/plugins/extraction/scheme.mli b/plugins/extraction/scheme.mli index b0fa395c6..51c73ef14 100644 --- a/plugins/extraction/scheme.mli +++ b/plugins/extraction/scheme.mli @@ -6,6 +6,4 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - val scheme_descr : Miniml.language_descr diff --git a/plugins/extraction/table.ml b/plugins/extraction/table.ml index 866f499b5..36ba0cd7d 100644 --- a/plugins/extraction/table.ml +++ b/plugins/extraction/table.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/plugins/extraction/table.mli b/plugins/extraction/table.mli index 512ecca74..b8cdea3b6 100644 --- a/plugins/extraction/table.mli +++ b/plugins/extraction/table.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Libnames open Miniml diff --git a/plugins/field/LegacyField.v b/plugins/field/LegacyField.v index efa53b4e9..bbc1e20b0 100644 --- a/plugins/field/LegacyField.v +++ b/plugins/field/LegacyField.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export LegacyField_Compl. Require Export LegacyField_Theory. Require Export LegacyField_Tactic. diff --git a/plugins/field/LegacyField_Compl.v b/plugins/field/LegacyField_Compl.v index d4a39296a..1df77ef09 100644 --- a/plugins/field/LegacyField_Compl.v +++ b/plugins/field/LegacyField_Compl.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import List. Definition assoc_2nd := diff --git a/plugins/field/LegacyField_Tactic.v b/plugins/field/LegacyField_Tactic.v index 5c1f228ac..50305d4a3 100644 --- a/plugins/field/LegacyField_Tactic.v +++ b/plugins/field/LegacyField_Tactic.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import List. Require Import LegacyRing. Require Export LegacyField_Compl. diff --git a/plugins/field/LegacyField_Theory.v b/plugins/field/LegacyField_Theory.v index cc8b043fc..907b137a3 100644 --- a/plugins/field/LegacyField_Theory.v +++ b/plugins/field/LegacyField_Theory.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import List. Require Import Peano_dec. Require Import LegacyRing. diff --git a/plugins/field/field.ml4 b/plugins/field/field.ml4 index 91c0ca21e..f08ed7db6 100644 --- a/plugins/field/field.ml4 +++ b/plugins/field/field.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Names open Pp open Proof_type diff --git a/plugins/firstorder/formula.ml b/plugins/firstorder/formula.ml index 45365cb2c..3a2ca70b6 100644 --- a/plugins/firstorder/formula.ml +++ b/plugins/firstorder/formula.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Hipattern open Names open Term diff --git a/plugins/firstorder/formula.mli b/plugins/firstorder/formula.mli index 2e89ddb06..77bc481a6 100644 --- a/plugins/firstorder/formula.mli +++ b/plugins/firstorder/formula.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Names open Libnames diff --git a/plugins/firstorder/g_ground.ml4 b/plugins/firstorder/g_ground.ml4 index f85616279..77f15aa07 100644 --- a/plugins/firstorder/g_ground.ml4 +++ b/plugins/firstorder/g_ground.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Formula open Sequent open Ground diff --git a/plugins/firstorder/ground.ml b/plugins/firstorder/ground.ml index 7f4acb856..1d9b0c79a 100644 --- a/plugins/firstorder/ground.ml +++ b/plugins/firstorder/ground.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Formula open Sequent open Rules diff --git a/plugins/firstorder/ground.mli b/plugins/firstorder/ground.mli index 3c0e903fd..6722a7935 100644 --- a/plugins/firstorder/ground.mli +++ b/plugins/firstorder/ground.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - val ground_tac: Tacmach.tactic -> (Proof_type.goal Tacmach.sigma -> Sequent.t) -> Tacmach.tactic diff --git a/plugins/firstorder/instances.ml b/plugins/firstorder/instances.ml index 810262a69..b473e5946 100644 --- a/plugins/firstorder/instances.ml +++ b/plugins/firstorder/instances.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Formula open Sequent open Unify diff --git a/plugins/firstorder/instances.mli b/plugins/firstorder/instances.mli index 95dd22ea8..43a1b746c 100644 --- a/plugins/firstorder/instances.mli +++ b/plugins/firstorder/instances.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Term open Tacmach open Names diff --git a/plugins/firstorder/rules.ml b/plugins/firstorder/rules.ml index 515efea70..fcc0f069b 100644 --- a/plugins/firstorder/rules.ml +++ b/plugins/firstorder/rules.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/plugins/firstorder/rules.mli b/plugins/firstorder/rules.mli index fc32621ca..c5498fe0a 100644 --- a/plugins/firstorder/rules.mli +++ b/plugins/firstorder/rules.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Tacmach open Names diff --git a/plugins/firstorder/sequent.ml b/plugins/firstorder/sequent.ml index 685d44a84..2f924198c 100644 --- a/plugins/firstorder/sequent.ml +++ b/plugins/firstorder/sequent.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Util open Formula diff --git a/plugins/firstorder/sequent.mli b/plugins/firstorder/sequent.mli index ce0eddccc..5e9f46aa2 100644 --- a/plugins/firstorder/sequent.mli +++ b/plugins/firstorder/sequent.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Util open Formula diff --git a/plugins/firstorder/unify.ml b/plugins/firstorder/unify.ml index e3a4c6a55..880e9a7d6 100644 --- a/plugins/firstorder/unify.ml +++ b/plugins/firstorder/unify.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Formula open Tacmach diff --git a/plugins/firstorder/unify.mli b/plugins/firstorder/unify.mli index d6cb3a082..60abdcd1a 100644 --- a/plugins/firstorder/unify.mli +++ b/plugins/firstorder/unify.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term exception UFAIL of constr*constr diff --git a/plugins/fourier/Fourier.v b/plugins/fourier/Fourier.v index 07b2973a4..dc971aacf 100644 --- a/plugins/fourier/Fourier.v +++ b/plugins/fourier/Fourier.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* "Fourier's method to solve linear inequations/equations systems.".*) Require Export LegacyRing. diff --git a/plugins/fourier/Fourier_util.v b/plugins/fourier/Fourier_util.v index 0fd92d606..1974e51ab 100644 --- a/plugins/fourier/Fourier_util.v +++ b/plugins/fourier/Fourier_util.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Rbase. Comments "Lemmas used by the tactic Fourier". diff --git a/plugins/fourier/fourier.ml b/plugins/fourier/fourier.ml index 73fb49295..21a5cb87f 100644 --- a/plugins/fourier/fourier.ml +++ b/plugins/fourier/fourier.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Méthode d'élimination de Fourier *) (* Référence: Auteur(s) : Fourier, Jean-Baptiste-Joseph diff --git a/plugins/fourier/fourierR.ml b/plugins/fourier/fourierR.ml index 3f490babd..dc6463f42 100644 --- a/plugins/fourier/fourierR.ml +++ b/plugins/fourier/fourierR.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* La tactique Fourier ne fonctionne de manière sûre que si les coefficients diff --git a/plugins/fourier/g_fourier.ml4 b/plugins/fourier/g_fourier.ml4 index b952851fa..705cc69e6 100644 --- a/plugins/fourier/g_fourier.ml4 +++ b/plugins/fourier/g_fourier.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open FourierR TACTIC EXTEND fourier diff --git a/plugins/funind/merge.ml b/plugins/funind/merge.ml index c69e04b93..26f49f6d4 100644 --- a/plugins/funind/merge.ml +++ b/plugins/funind/merge.ml @@ -8,7 +8,6 @@ (* Merging of induction principles. *) -(*i $Id: i*) open Libnames open Tactics open Indfun_common diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml index 8dc660b42..1780ff827 100644 --- a/plugins/funind/recdef.ml +++ b/plugins/funind/recdef.ml @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Term open Termops open Namegen diff --git a/plugins/micromega/g_micromega.ml4 b/plugins/micromega/g_micromega.ml4 index f4d04e5d4..869ce84b9 100644 --- a/plugins/micromega/g_micromega.ml4 +++ b/plugins/micromega/g_micromega.ml4 @@ -14,8 +14,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Quote open Ring open Mutils diff --git a/plugins/omega/Omega.v b/plugins/omega/Omega.v index 30b945718..6d0b6bae1 100644 --- a/plugins/omega/Omega.v +++ b/plugins/omega/Omega.v @@ -13,8 +13,6 @@ (* *) (**************************************************************************) -(* $Id$ *) - (* We do not require [ZArith] anymore, but only what's necessary for Omega *) Require Export ZArith_base. Require Export OmegaLemmas. diff --git a/plugins/omega/OmegaLemmas.v b/plugins/omega/OmegaLemmas.v index 56a854d6f..ff433bbd8 100644 --- a/plugins/omega/OmegaLemmas.v +++ b/plugins/omega/OmegaLemmas.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(*i $Id$ i*) - Require Import ZArith_base. Open Local Scope Z_scope. diff --git a/plugins/omega/OmegaPlugin.v b/plugins/omega/OmegaPlugin.v index 21535f0d3..9ec850c0b 100644 --- a/plugins/omega/OmegaPlugin.v +++ b/plugins/omega/OmegaPlugin.v @@ -6,6 +6,4 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Declare ML Module "omega_plugin". diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml index 60616845b..da2f27994 100644 --- a/plugins/omega/coq_omega.ml +++ b/plugins/omega/coq_omega.ml @@ -13,8 +13,6 @@ (* *) (**************************************************************************) -(* $Id$ *) - open Util open Pp open Reduction diff --git a/plugins/omega/g_omega.ml4 b/plugins/omega/g_omega.ml4 index 3bfdce7fd..7751d767b 100644 --- a/plugins/omega/g_omega.ml4 +++ b/plugins/omega/g_omega.ml4 @@ -15,8 +15,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Coq_omega open Refiner diff --git a/plugins/quote/Quote.v b/plugins/quote/Quote.v index 11726675b..bb90f7f57 100644 --- a/plugins/quote/Quote.v +++ b/plugins/quote/Quote.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Declare ML Module "quote_plugin". (*********************************************************************** diff --git a/plugins/quote/g_quote.ml4 b/plugins/quote/g_quote.ml4 index bdeb9844b..216b7840f 100644 --- a/plugins/quote/g_quote.ml4 +++ b/plugins/quote/g_quote.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Util open Tacexpr open Quote diff --git a/plugins/quote/quote.ml b/plugins/quote/quote.ml index ce65a45ec..6d096beec 100644 --- a/plugins/quote/quote.ml +++ b/plugins/quote/quote.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* The `Quote' tactic *) (* The basic idea is to automatize the inversion of interpetation functions diff --git a/plugins/ring/LegacyArithRing.v b/plugins/ring/LegacyArithRing.v index 231b5fbb0..9572c1ce7 100644 --- a/plugins/ring/LegacyArithRing.v +++ b/plugins/ring/LegacyArithRing.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Instantiation of the Ring tactic for the naturals of Arith $*) Require Import Bool. diff --git a/plugins/ring/LegacyNArithRing.v b/plugins/ring/LegacyNArithRing.v index ee9fb3761..eb62def87 100644 --- a/plugins/ring/LegacyNArithRing.v +++ b/plugins/ring/LegacyNArithRing.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Instantiation of the Ring tactic for the binary natural numbers *) Require Import Bool. diff --git a/plugins/ring/LegacyRing.v b/plugins/ring/LegacyRing.v index 4ae85baf3..cd51f9e02 100644 --- a/plugins/ring/LegacyRing.v +++ b/plugins/ring/LegacyRing.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Bool. Require Export LegacyRing_theory. Require Export Quote. diff --git a/plugins/ring/LegacyRing_theory.v b/plugins/ring/LegacyRing_theory.v index 30d29515f..a3071f7b4 100644 --- a/plugins/ring/LegacyRing_theory.v +++ b/plugins/ring/LegacyRing_theory.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Bool. Set Implicit Arguments. diff --git a/plugins/ring/LegacyZArithRing.v b/plugins/ring/LegacyZArithRing.v index 68a0dd275..c48d61b0d 100644 --- a/plugins/ring/LegacyZArithRing.v +++ b/plugins/ring/LegacyZArithRing.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Instantiation of the Ring tactic for the binary integers of ZArith *) Require Export LegacyArithRing. diff --git a/plugins/ring/Ring_abstract.v b/plugins/ring/Ring_abstract.v index 2a9df21b3..cccfe653b 100644 --- a/plugins/ring/Ring_abstract.v +++ b/plugins/ring/Ring_abstract.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import LegacyRing_theory. Require Import Quote. Require Import Ring_normalize. diff --git a/plugins/ring/Ring_normalize.v b/plugins/ring/Ring_normalize.v index 7aeee2185..54ddcb9ae 100644 --- a/plugins/ring/Ring_normalize.v +++ b/plugins/ring/Ring_normalize.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import LegacyRing_theory. Require Import Quote. diff --git a/plugins/ring/Setoid_ring.v b/plugins/ring/Setoid_ring.v index 93b9bc7cf..127228116 100644 --- a/plugins/ring/Setoid_ring.v +++ b/plugins/ring/Setoid_ring.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Setoid_ring_theory. Require Export Quote. Require Export Setoid_ring_normalize. diff --git a/plugins/ring/Setoid_ring_normalize.v b/plugins/ring/Setoid_ring_normalize.v index 9b4c46fe9..8d77854b6 100644 --- a/plugins/ring/Setoid_ring_normalize.v +++ b/plugins/ring/Setoid_ring_normalize.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import Setoid_ring_theory. Require Import Quote. diff --git a/plugins/ring/Setoid_ring_theory.v b/plugins/ring/Setoid_ring_theory.v index 2c2314aff..0444fe74a 100644 --- a/plugins/ring/Setoid_ring_theory.v +++ b/plugins/ring/Setoid_ring_theory.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Bool. Require Export Setoid. diff --git a/plugins/ring/g_ring.ml4 b/plugins/ring/g_ring.ml4 index d766e3445..99650a32f 100644 --- a/plugins/ring/g_ring.ml4 +++ b/plugins/ring/g_ring.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Quote open Ring open Tacticals diff --git a/plugins/ring/ring.ml b/plugins/ring/ring.ml index fdf3a9bd9..81f6b66ee 100644 --- a/plugins/ring/ring.ml +++ b/plugins/ring/ring.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* ML part of the Ring tactic *) open Pp diff --git a/plugins/rtauto/Bintree.v b/plugins/rtauto/Bintree.v index 36da9463b..598b21d83 100644 --- a/plugins/rtauto/Bintree.v +++ b/plugins/rtauto/Bintree.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export List. Require Export BinPos. diff --git a/plugins/rtauto/Rtauto.v b/plugins/rtauto/Rtauto.v index 0d1d09c73..47fc11825 100644 --- a/plugins/rtauto/Rtauto.v +++ b/plugins/rtauto/Rtauto.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export List. Require Export Bintree. diff --git a/plugins/rtauto/g_rtauto.ml4 b/plugins/rtauto/g_rtauto.ml4 index 4cbe84368..6309a7425 100644 --- a/plugins/rtauto/g_rtauto.ml4 +++ b/plugins/rtauto/g_rtauto.ml4 @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$*) - (*i camlp4deps: "parsing/grammar.cma" i*) TACTIC EXTEND rtauto diff --git a/plugins/rtauto/proof_search.ml b/plugins/rtauto/proof_search.ml index 562e2e3bd..029e7eafd 100644 --- a/plugins/rtauto/proof_search.ml +++ b/plugins/rtauto/proof_search.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Util open Goptions diff --git a/plugins/rtauto/proof_search.mli b/plugins/rtauto/proof_search.mli index e52f6bbdc..44a5f49c6 100644 --- a/plugins/rtauto/proof_search.mli +++ b/plugins/rtauto/proof_search.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - type form= Atom of int | Arrow of form * form diff --git a/plugins/rtauto/refl_tauto.ml b/plugins/rtauto/refl_tauto.ml index 06313e8fe..3ae25da65 100644 --- a/plugins/rtauto/refl_tauto.ml +++ b/plugins/rtauto/refl_tauto.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - module Search = Explore.Make(Proof_search) open Util diff --git a/plugins/rtauto/refl_tauto.mli b/plugins/rtauto/refl_tauto.mli index a6d68a226..79872f2cd 100644 --- a/plugins/rtauto/refl_tauto.mli +++ b/plugins/rtauto/refl_tauto.mli @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* raises Not_found if no proof is found *) type atom_env= diff --git a/plugins/setoid_ring/newring.ml4 b/plugins/setoid_ring/newring.ml4 index d6dece458..0f8c2f010 100644 --- a/plugins/setoid_ring/newring.ml4 +++ b/plugins/setoid_ring/newring.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/plugins/subtac/eterm.mli b/plugins/subtac/eterm.mli index 406f94338..0dfeca511 100644 --- a/plugins/subtac/eterm.mli +++ b/plugins/subtac/eterm.mli @@ -6,7 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) open Environ open Tacmach open Term diff --git a/plugins/subtac/g_subtac.ml4 b/plugins/subtac/g_subtac.ml4 index 700e61911..28ded30da 100644 --- a/plugins/subtac/g_subtac.ml4 +++ b/plugins/subtac/g_subtac.ml4 @@ -14,8 +14,6 @@ Syntax for the subtac terms and types. Elaborated from correctness/psyntax.ml4 by Jean-Christophe Filliâtre *) -(* $Id$ *) - open Flags open Util diff --git a/plugins/subtac/subtac.ml b/plugins/subtac/subtac.ml index e649ad97b..569aba263 100644 --- a/plugins/subtac/subtac.ml +++ b/plugins/subtac/subtac.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Global open Pp open Util diff --git a/plugins/subtac/subtac_cases.ml b/plugins/subtac/subtac_cases.ml index 60e8cb0f7..4ec34a91a 100644 --- a/plugins/subtac/subtac_cases.ml +++ b/plugins/subtac/subtac_cases.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Cases open Util open Names diff --git a/plugins/subtac/subtac_cases.mli b/plugins/subtac/subtac_cases.mli index 90989d2d3..4636bddc0 100644 --- a/plugins/subtac/subtac_cases.mli +++ b/plugins/subtac/subtac_cases.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/plugins/subtac/subtac_classes.ml b/plugins/subtac/subtac_classes.ml index 5c9deab8d..07b076e67 100644 --- a/plugins/subtac/subtac_classes.ml +++ b/plugins/subtac/subtac_classes.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pretyping open Evd open Environ diff --git a/plugins/subtac/subtac_classes.mli b/plugins/subtac/subtac_classes.mli index ee78ff68a..6478d2065 100644 --- a/plugins/subtac/subtac_classes.mli +++ b/plugins/subtac/subtac_classes.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Decl_kinds diff --git a/plugins/subtac/subtac_coercion.ml b/plugins/subtac/subtac_coercion.ml index 9161d8887..6b07e3591 100644 --- a/plugins/subtac/subtac_coercion.ml +++ b/plugins/subtac/subtac_coercion.ml @@ -6,8 +6,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/plugins/subtac/subtac_pretyping.ml b/plugins/subtac/subtac_pretyping.ml index 775397124..76229076c 100644 --- a/plugins/subtac/subtac_pretyping.ml +++ b/plugins/subtac/subtac_pretyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Global open Pp open Util diff --git a/plugins/subtac/subtac_pretyping_F.ml b/plugins/subtac/subtac_pretyping_F.ml index b49190d44..4d7bcb1eb 100644 --- a/plugins/subtac/subtac_pretyping_F.ml +++ b/plugins/subtac/subtac_pretyping_F.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/plugins/syntax/ascii_syntax.ml b/plugins/syntax/ascii_syntax.ml index 19473dfa6..79e1a6eb2 100644 --- a/plugins/syntax/ascii_syntax.ml +++ b/plugins/syntax/ascii_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/plugins/syntax/nat_syntax.ml b/plugins/syntax/nat_syntax.ml index 5d20c2a3c..932b20f38 100644 --- a/plugins/syntax/nat_syntax.ml +++ b/plugins/syntax/nat_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* This file defines the printer for natural numbers in [nat] *) (*i*) diff --git a/plugins/syntax/numbers_syntax.ml b/plugins/syntax/numbers_syntax.ml index 4375d5e0f..826b5c384 100644 --- a/plugins/syntax/numbers_syntax.ml +++ b/plugins/syntax/numbers_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* digit-based syntax for int31, bigN bigZ and bigQ *) open Bigint diff --git a/plugins/syntax/r_syntax.ml b/plugins/syntax/r_syntax.ml index f85309e67..38e0a159f 100644 --- a/plugins/syntax/r_syntax.ml +++ b/plugins/syntax/r_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/plugins/syntax/string_syntax.ml b/plugins/syntax/string_syntax.ml index bc02357ae..cb2b16858 100644 --- a/plugins/syntax/string_syntax.ml +++ b/plugins/syntax/string_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/plugins/syntax/z_syntax.ml b/plugins/syntax/z_syntax.ml index f6afd080f..7d5ee96d1 100644 --- a/plugins/syntax/z_syntax.ml +++ b/plugins/syntax/z_syntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pcoq open Pp open Util diff --git a/plugins/xml/xml.mli b/plugins/xml/xml.mli index 3775287a5..195b37bbc 100644 --- a/plugins/xml/xml.mli +++ b/plugins/xml/xml.mli @@ -12,8 +12,6 @@ (* http://helm.cs.unibo.it *) (************************************************************************) -(*i $Id$ i*) - (* Tokens for XML cdata, empty elements and not-empty elements *) (* Usage: *) (* Str cdata *) diff --git a/plugins/xml/xmlcommand.mli b/plugins/xml/xmlcommand.mli index 66ff9f0bb..1a6aea97b 100644 --- a/plugins/xml/xmlcommand.mli +++ b/plugins/xml/xmlcommand.mli @@ -12,8 +12,6 @@ (* http://helm.cs.unibo.it *) (************************************************************************) -(*i $Id$ i*) - (* print_global qid fn *) (* where qid is a long name denoting a definition/theorem or *) (* an inductive definition *) diff --git a/plugins/xml/xmlentries.ml4 b/plugins/xml/xmlentries.ml4 index 41c107ad2..ec1613144 100644 --- a/plugins/xml/xmlentries.ml4 +++ b/plugins/xml/xmlentries.ml4 @@ -14,8 +14,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Util;; open Vernacinterp;; diff --git a/pretyping/cases.ml b/pretyping/cases.ml index f68bf10c4..4b565ddbd 100644 --- a/pretyping/cases.ml +++ b/pretyping/cases.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Nameops diff --git a/pretyping/cases.mli b/pretyping/cases.mli index 188959f6a..202a794ab 100644 --- a/pretyping/cases.mli +++ b/pretyping/cases.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/pretyping/cbv.ml b/pretyping/cbv.ml index 8c03d0df4..8a7182708 100644 --- a/pretyping/cbv.ml +++ b/pretyping/cbv.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Term diff --git a/pretyping/cbv.mli b/pretyping/cbv.mli index 75017d5b4..50b4fda4a 100644 --- a/pretyping/cbv.mli +++ b/pretyping/cbv.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/pretyping/classops.ml b/pretyping/classops.ml index 237963258..5c30f05aa 100644 --- a/pretyping/classops.ml +++ b/pretyping/classops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Flags diff --git a/pretyping/classops.mli b/pretyping/classops.mli index 1830df3fb..890aa005c 100644 --- a/pretyping/classops.mli +++ b/pretyping/classops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Decl_kinds open Term diff --git a/pretyping/coercion.ml b/pretyping/coercion.ml index 3607362a6..f2975d21c 100644 --- a/pretyping/coercion.ml +++ b/pretyping/coercion.ml @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/pretyping/coercion.mli b/pretyping/coercion.mli index 3ac83fc19..a5ed740f9 100644 --- a/pretyping/coercion.mli +++ b/pretyping/coercion.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Evd open Names diff --git a/pretyping/detyping.ml b/pretyping/detyping.ml index 6560f7b48..9113efd55 100644 --- a/pretyping/detyping.ml +++ b/pretyping/detyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Univ diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli index 7b14c4fd2..47a7beb53 100644 --- a/pretyping/detyping.mli +++ b/pretyping/detyping.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/pretyping/evarconv.ml b/pretyping/evarconv.ml index b43e6e999..4b76b7709 100644 --- a/pretyping/evarconv.ml +++ b/pretyping/evarconv.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/evarconv.mli b/pretyping/evarconv.mli index 2e52fb12b..8ea91d28f 100644 --- a/pretyping/evarconv.mli +++ b/pretyping/evarconv.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Sign open Environ diff --git a/pretyping/evarutil.ml b/pretyping/evarutil.ml index 6d37cf80f..fbfb33cc3 100644 --- a/pretyping/evarutil.ml +++ b/pretyping/evarutil.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/pretyping/evarutil.mli b/pretyping/evarutil.mli index 3f66dc97e..de50a8761 100644 --- a/pretyping/evarutil.mli +++ b/pretyping/evarutil.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Rawterm diff --git a/pretyping/evd.ml b/pretyping/evd.ml index 5b4a3f214..61a0353dd 100644 --- a/pretyping/evd.ml +++ b/pretyping/evd.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/evd.mli b/pretyping/evd.mli index 2601d44f7..ebf91b4f4 100644 --- a/pretyping/evd.mli +++ b/pretyping/evd.mli @@ -7,8 +7,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/pretyping/indrec.ml b/pretyping/indrec.ml index 1352b3830..1daae0236 100644 --- a/pretyping/indrec.ml +++ b/pretyping/indrec.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* File initially created by Christine Paulin, 1996 *) (* This file builds various inductive schemes *) diff --git a/pretyping/indrec.mli b/pretyping/indrec.mli index 304b986a1..7f19c5d37 100644 --- a/pretyping/indrec.mli +++ b/pretyping/indrec.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/pretyping/inductiveops.ml b/pretyping/inductiveops.ml index 3897b18e5..07447c540 100644 --- a/pretyping/inductiveops.ml +++ b/pretyping/inductiveops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Univ diff --git a/pretyping/inductiveops.mli b/pretyping/inductiveops.mli index 6255a83d4..98a22fabd 100644 --- a/pretyping/inductiveops.mli +++ b/pretyping/inductiveops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Declarations diff --git a/pretyping/matching.ml b/pretyping/matching.ml index b94642c09..2c0285ed2 100644 --- a/pretyping/matching.ml +++ b/pretyping/matching.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Util open Names diff --git a/pretyping/matching.mli b/pretyping/matching.mli index 263ded381..95314054e 100644 --- a/pretyping/matching.mli +++ b/pretyping/matching.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/pretyping/namegen.ml b/pretyping/namegen.ml index 7d141faf1..7f0b14f06 100644 --- a/pretyping/namegen.ml +++ b/pretyping/namegen.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Created from contents that was formerly in termops.ml and nameops.ml, Nov 2009 *) diff --git a/pretyping/namegen.mli b/pretyping/namegen.mli index e3ab7d03e..889f8ec8c 100644 --- a/pretyping/namegen.mli +++ b/pretyping/namegen.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: namegen.mli 12549 2009-12-01 12:05:57Z herbelin {% $ %} *) - open Names open Term open Environ diff --git a/pretyping/pattern.ml b/pretyping/pattern.ml index f9dec8f35..48218f47f 100644 --- a/pretyping/pattern.ml +++ b/pretyping/pattern.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Libnames diff --git a/pretyping/pattern.mli b/pretyping/pattern.mli index 33105c312..d805730e9 100644 --- a/pretyping/pattern.mli +++ b/pretyping/pattern.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names open Sign diff --git a/pretyping/pretype_errors.ml b/pretyping/pretype_errors.ml index 2f7a7c87c..6adaee81c 100644 --- a/pretyping/pretype_errors.ml +++ b/pretyping/pretype_errors.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Stdpp open Names diff --git a/pretyping/pretype_errors.mli b/pretyping/pretype_errors.mli index 9b6216a12..e6e01fc44 100644 --- a/pretyping/pretype_errors.mli +++ b/pretyping/pretype_errors.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/pretyping/pretyping.ml b/pretyping/pretyping.ml index 8654ca947..92968cad9 100644 --- a/pretyping/pretyping.ml +++ b/pretyping/pretyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/pretyping.mli b/pretyping/pretyping.mli index f5601d6d6..eba26bafe 100644 --- a/pretyping/pretyping.mli +++ b/pretyping/pretyping.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Sign open Term diff --git a/pretyping/rawterm.ml b/pretyping/rawterm.ml index 16421b2a7..784e6b6e0 100644 --- a/pretyping/rawterm.ml +++ b/pretyping/rawterm.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (*i*) open Util open Names diff --git a/pretyping/rawterm.mli b/pretyping/rawterm.mli index ac4f0dec6..9e2d1f28c 100644 --- a/pretyping/rawterm.mli +++ b/pretyping/rawterm.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/pretyping/recordops.ml b/pretyping/recordops.ml index d94da115a..32433f6be 100644 --- a/pretyping/recordops.ml +++ b/pretyping/recordops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/pretyping/recordops.mli b/pretyping/recordops.mli index 954890d89..78b01eeab 100755 --- a/pretyping/recordops.mli +++ b/pretyping/recordops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Nametab open Term diff --git a/pretyping/reductionops.ml b/pretyping/reductionops.ml index b741c9a41..dae668243 100644 --- a/pretyping/reductionops.ml +++ b/pretyping/reductionops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/reductionops.mli b/pretyping/reductionops.mli index 84bd20135..f3bfa1e5f 100644 --- a/pretyping/reductionops.mli +++ b/pretyping/reductionops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Univ diff --git a/pretyping/retyping.ml b/pretyping/retyping.ml index 1e0649da6..db0ee942a 100644 --- a/pretyping/retyping.ml +++ b/pretyping/retyping.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Term open Inductive diff --git a/pretyping/retyping.mli b/pretyping/retyping.mli index 3c68f850b..5b445ff9c 100644 --- a/pretyping/retyping.mli +++ b/pretyping/retyping.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Evd diff --git a/pretyping/tacred.ml b/pretyping/tacred.ml index a103c49b6..6dbbff170 100644 --- a/pretyping/tacred.ml +++ b/pretyping/tacred.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/tacred.mli b/pretyping/tacred.mli index 84cff15b6..fdceadfbb 100644 --- a/pretyping/tacred.mli +++ b/pretyping/tacred.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/pretyping/term_dnet.ml b/pretyping/term_dnet.ml index 04e328cbd..c7cfaed4b 100644 --- a/pretyping/term_dnet.ml +++ b/pretyping/term_dnet.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id:$ *) - (*i*) open Util open Term diff --git a/pretyping/term_dnet.mli b/pretyping/term_dnet.mli index 7623fcd68..3db55b162 100644 --- a/pretyping/term_dnet.mli +++ b/pretyping/term_dnet.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id:{% $ %} *) - open Term open Sign open Libnames diff --git a/pretyping/termops.ml b/pretyping/termops.ml index 4de4bde2c..1c0bf2fbc 100644 --- a/pretyping/termops.ml +++ b/pretyping/termops.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/termops.mli b/pretyping/termops.mli index 57b5bd581..9f3884088 100644 --- a/pretyping/termops.mli +++ b/pretyping/termops.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Pp open Names diff --git a/pretyping/typeclasses.ml b/pretyping/typeclasses.ml index 88d4a4d6b..2a716ee6a 100644 --- a/pretyping/typeclasses.ml +++ b/pretyping/typeclasses.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Libnames diff --git a/pretyping/typeclasses.mli b/pretyping/typeclasses.mli index c816f2e9c..dc1c5f556 100644 --- a/pretyping/typeclasses.mli +++ b/pretyping/typeclasses.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Libnames open Decl_kinds diff --git a/pretyping/typeclasses_errors.ml b/pretyping/typeclasses_errors.ml index 1de8b7a5f..869a7845d 100644 --- a/pretyping/typeclasses_errors.ml +++ b/pretyping/typeclasses_errors.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Decl_kinds diff --git a/pretyping/typeclasses_errors.mli b/pretyping/typeclasses_errors.mli index 24a19a0e3..43b349515 100644 --- a/pretyping/typeclasses_errors.mli +++ b/pretyping/typeclasses_errors.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Decl_kinds open Term diff --git a/pretyping/typing.ml b/pretyping/typing.ml index 831787a06..8670b95f9 100644 --- a/pretyping/typing.ml +++ b/pretyping/typing.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/pretyping/typing.mli b/pretyping/typing.mli index c20fd9453..90f823b8e 100644 --- a/pretyping/typing.mli +++ b/pretyping/typing.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Environ open Evd diff --git a/pretyping/unification.ml b/pretyping/unification.ml index 35543ce24..7ae05a85f 100644 --- a/pretyping/unification.ml +++ b/pretyping/unification.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/pretyping/unification.mli b/pretyping/unification.mli index 13042180a..8829d8989 100644 --- a/pretyping/unification.mli +++ b/pretyping/unification.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Environ open Evd diff --git a/pretyping/vnorm.ml b/pretyping/vnorm.ml index c894d2b51..7e41e2125 100644 --- a/pretyping/vnorm.ml +++ b/pretyping/vnorm.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Declarations open Term diff --git a/proofs/clenv.ml b/proofs/clenv.ml index 35db5e6ed..006892189 100644 --- a/proofs/clenv.ml +++ b/proofs/clenv.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/clenv.mli b/proofs/clenv.mli index a97b85ed9..afda6d931 100644 --- a/proofs/clenv.mli +++ b/proofs/clenv.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/proofs/clenvtac.ml b/proofs/clenvtac.ml index f977768bd..a8162cc5a 100644 --- a/proofs/clenvtac.ml +++ b/proofs/clenvtac.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/clenvtac.mli b/proofs/clenvtac.mli index 02bf86641..760a79d4c 100644 --- a/proofs/clenvtac.mli +++ b/proofs/clenvtac.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/proofs/evar_refiner.ml b/proofs/evar_refiner.ml index 6dfbbdc12..cd05cdcd2 100644 --- a/proofs/evar_refiner.ml +++ b/proofs/evar_refiner.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/proofs/evar_refiner.mli b/proofs/evar_refiner.mli index ff986f3e6..ca3bd1e80 100644 --- a/proofs/evar_refiner.mli +++ b/proofs/evar_refiner.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Environ diff --git a/proofs/goal.ml b/proofs/goal.ml index a9202318d..4e5905d83 100644 --- a/proofs/goal.ml +++ b/proofs/goal.ml @@ -6,8 +6,6 @@ (* * GNU Lesscer General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term (* This module implements the abstract interface to goals *) diff --git a/proofs/goal.mli b/proofs/goal.mli index 49e3c9b1a..c7f695766 100644 --- a/proofs/goal.mli +++ b/proofs/goal.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: goal.mli aspiwack $ *) - (* This module implements the abstract interface to goals *) type goal diff --git a/proofs/logic.ml b/proofs/logic.ml index 7c092bb66..93de5be69 100644 --- a/proofs/logic.ml +++ b/proofs/logic.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/logic.mli b/proofs/logic.mli index eec3de730..39f69ad12 100644 --- a/proofs/logic.mli +++ b/proofs/logic.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Sign diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml index 6da73c2f6..153354c92 100644 --- a/proofs/pfedit.ml +++ b/proofs/pfedit.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli index 47b741f5d..194dd1464 100644 --- a/proofs/pfedit.mli +++ b/proofs/pfedit.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Pp open Names diff --git a/proofs/proof.ml b/proofs/proof.ml index 0c298cc63..35f7b4f02 100644 --- a/proofs/proof.ml +++ b/proofs/proof.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Module defining the last essential tiles of interactive proofs. The features of the Proof module are undoing and focusing. A proof is a mutable object, it contains a proofview, and some information diff --git a/proofs/proof.mli b/proofs/proof.mli index 2b1c3f5c2..5e1120f9c 100644 --- a/proofs/proof.mli +++ b/proofs/proof.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: proof.mli aspiwack $ *) - (* Module defining the last essential tiles of interactive proofs. The features of the Proof module are undoing and focusing. A proof is a mutable object, it contains a proofview, and some information diff --git a/proofs/proof_global.ml b/proofs/proof_global.ml index 420ff8432..87a8d8d1e 100644 --- a/proofs/proof_global.ml +++ b/proofs/proof_global.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (***********************************************************************) (* *) (* This module defines the global proof environment *) diff --git a/proofs/proof_global.mli b/proofs/proof_global.mli index 84a61c755..40908dfc4 100644 --- a/proofs/proof_global.mli +++ b/proofs/proof_global.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (***********************************************************************) (* *) (* This module defines the global proof environment *) diff --git a/proofs/proof_type.ml b/proofs/proof_type.ml index 2fffa3952..55a73c608 100644 --- a/proofs/proof_type.ml +++ b/proofs/proof_type.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ *) - (*i*) open Environ open Evd diff --git a/proofs/proof_type.mli b/proofs/proof_type.mli index 7d8875302..8def61112 100644 --- a/proofs/proof_type.mli +++ b/proofs/proof_type.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Environ open Evd open Names diff --git a/proofs/proofview.ml b/proofs/proofview.ml index a08941df0..427a8d613 100644 --- a/proofs/proofview.ml +++ b/proofs/proofview.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* The proofview datastructure is a pure datastructure underlying the notion of proof (namely, a proof is a proofview which can evolve and has safety mechanisms attached). diff --git a/proofs/proofview.mli b/proofs/proofview.mli index cd5520d4e..dc205f538 100644 --- a/proofs/proofview.mli +++ b/proofs/proofview.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: proofview.mli aspiwack $ *) - (* The proofview datastructure is a pure datastructure underlying the notion of proof (namely, a proof is a proofview which can evolve and has safety mechanisms attached). diff --git a/proofs/redexpr.ml b/proofs/redexpr.ml index b0a01caa7..b30097731 100644 --- a/proofs/redexpr.ml +++ b/proofs/redexpr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/redexpr.mli b/proofs/redexpr.mli index 199130b5f..581ee1dc9 100644 --- a/proofs/redexpr.mli +++ b/proofs/redexpr.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Closure diff --git a/proofs/refiner.ml b/proofs/refiner.ml index ffb18f265..1abd76253 100644 --- a/proofs/refiner.ml +++ b/proofs/refiner.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Term diff --git a/proofs/refiner.mli b/proofs/refiner.mli index 958560044..be4dbd9a5 100644 --- a/proofs/refiner.mli +++ b/proofs/refiner.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Sign open Evd diff --git a/proofs/tacexpr.ml b/proofs/tacexpr.ml index b56e5184e..4cec846fd 100644 --- a/proofs/tacexpr.ml +++ b/proofs/tacexpr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Topconstr open Libnames diff --git a/proofs/tacmach.ml b/proofs/tacmach.ml index 6dbdf17cb..810429519 100644 --- a/proofs/tacmach.ml +++ b/proofs/tacmach.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli index cf704d101..9e0ca2a3d 100644 --- a/proofs/tacmach.mli +++ b/proofs/tacmach.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Sign diff --git a/proofs/tactic_debug.ml b/proofs/tactic_debug.ml index f6b2ce452..a3fa59e8a 100644 --- a/proofs/tactic_debug.ml +++ b/proofs/tactic_debug.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Names open Constrextern open Pp diff --git a/proofs/tactic_debug.mli b/proofs/tactic_debug.mli index f27540315..ac3bf493a 100644 --- a/proofs/tactic_debug.mli +++ b/proofs/tactic_debug.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Environ open Pattern open Evd diff --git a/scripts/coqc.ml b/scripts/coqc.ml index 61f13d4d7..a7d3afdb1 100644 --- a/scripts/coqc.ml +++ b/scripts/coqc.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Afin de rendre Coq plus portable, ce programme Caml remplace le script coqc. diff --git a/scripts/coqmktop.ml b/scripts/coqmktop.ml index bd21c1c52..ea777e6c5 100644 --- a/scripts/coqmktop.ml +++ b/scripts/coqmktop.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* coqmktop is a script to link Coq, analogous to ocamlmktop. The command line contains options specific to coqmktop, options for the Ocaml linker and files to link (in addition to the default Coq files). *) diff --git a/tactics/auto.ml b/tactics/auto.ml index d2bb1a06f..32a199e60 100644 --- a/tactics/auto.ml +++ b/tactics/auto.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/auto.mli b/tactics/auto.mli index 37fe3d441..f7c3fd777 100644 --- a/tactics/auto.mli +++ b/tactics/auto.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/tactics/autorewrite.ml b/tactics/autorewrite.ml index a0dea0292..2b05fcb65 100644 --- a/tactics/autorewrite.ml +++ b/tactics/autorewrite.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Equality open Hipattern open Names diff --git a/tactics/autorewrite.mli b/tactics/autorewrite.mli index a9556891a..bda1fc65f 100644 --- a/tactics/autorewrite.mli +++ b/tactics/autorewrite.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Tacexpr open Tacmach diff --git a/tactics/btermdn.ml b/tactics/btermdn.ml index bcb9a411c..13027fd34 100644 --- a/tactics/btermdn.ml +++ b/tactics/btermdn.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Names open Termdn diff --git a/tactics/btermdn.mli b/tactics/btermdn.mli index ebb046a05..a4ace7637 100644 --- a/tactics/btermdn.mli +++ b/tactics/btermdn.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Pattern open Names diff --git a/tactics/class_tactics.ml4 b/tactics/class_tactics.ml4 index e0e7aae2f..18d2c6081 100644 --- a/tactics/class_tactics.ml4 +++ b/tactics/class_tactics.ml4 @@ -9,8 +9,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/contradiction.ml b/tactics/contradiction.ml index 46ed2134d..29604a95f 100644 --- a/tactics/contradiction.ml +++ b/tactics/contradiction.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Term open Proof_type diff --git a/tactics/contradiction.mli b/tactics/contradiction.mli index b5fdf5a1b..b74a23271 100644 --- a/tactics/contradiction.mli +++ b/tactics/contradiction.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Proof_type diff --git a/tactics/dhyp.ml b/tactics/dhyp.ml index 96d83b972..f45685eaf 100644 --- a/tactics/dhyp.ml +++ b/tactics/dhyp.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Chet's comments about this tactic : Programmable destruction of hypotheses and conclusions. diff --git a/tactics/dhyp.mli b/tactics/dhyp.mli index 465a2a377..c35b4d759 100644 --- a/tactics/dhyp.mli +++ b/tactics/dhyp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Tacmach open Tacexpr diff --git a/tactics/eauto.ml4 b/tactics/eauto.ml4 index 49af8b40e..ebef403a1 100644 --- a/tactics/eauto.ml4 +++ b/tactics/eauto.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/elim.ml b/tactics/elim.ml index cac200f58..7baa5cd8c 100644 --- a/tactics/elim.ml +++ b/tactics/elim.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/elim.mli b/tactics/elim.mli index 7fbb16ba1..2351947e0 100644 --- a/tactics/elim.mli +++ b/tactics/elim.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Proof_type diff --git a/tactics/elimschemes.ml b/tactics/elimschemes.ml index e3f29fe59..28c696010 100644 --- a/tactics/elimschemes.ml +++ b/tactics/elimschemes.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Created by Hugo Herbelin from contents related to inductive schemes initially developed by Christine Paulin (induction schemes), Vincent Siles (decidable equality and boolean equality) and Matthieu Sozeau diff --git a/tactics/elimschemes.mli b/tactics/elimschemes.mli index ef1c4ec3e..d58878838 100644 --- a/tactics/elimschemes.mli +++ b/tactics/elimschemes.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(** {% $ %}Id: elimschemes.mli 12584 2009-12-13 21:04:34Z herbelin {% $ %} *) - open Ind_tables (** Induction/recursion schemes *) diff --git a/tactics/eqdecide.ml4 b/tactics/eqdecide.ml4 index d5e4ca17d..a93be7bc6 100644 --- a/tactics/eqdecide.ml4 +++ b/tactics/eqdecide.ml4 @@ -14,8 +14,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Util open Names open Namegen diff --git a/tactics/eqschemes.ml b/tactics/eqschemes.ml index 51dbd7ecd..195d4b7c4 100644 --- a/tactics/eqschemes.ml +++ b/tactics/eqschemes.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* File created by Hugo Herbelin, Nov 2009 *) (* This file builds schemes related to equality inductive types, diff --git a/tactics/eqschemes.mli b/tactics/eqschemes.mli index bdf3bbe76..8c649aecf 100644 --- a/tactics/eqschemes.mli +++ b/tactics/eqschemes.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** This file builds schemes relative to equality inductive types *) open Names diff --git a/tactics/equality.ml b/tactics/equality.ml index 8a4fb392e..1a5a92fc3 100644 --- a/tactics/equality.ml +++ b/tactics/equality.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/equality.mli b/tactics/equality.mli index b5c147393..d5694ba89 100644 --- a/tactics/equality.mli +++ b/tactics/equality.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Util open Names diff --git a/tactics/evar_tactics.ml b/tactics/evar_tactics.ml index 906c32c57..c8e6c9769 100644 --- a/tactics/evar_tactics.ml +++ b/tactics/evar_tactics.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Util open Evar_refiner diff --git a/tactics/evar_tactics.mli b/tactics/evar_tactics.mli index 0cf4dbb80..ffce59547 100644 --- a/tactics/evar_tactics.mli +++ b/tactics/evar_tactics.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Tacmach open Names open Tacexpr diff --git a/tactics/extraargs.ml4 b/tactics/extraargs.ml4 index adf8275ee..dd37822a1 100644 --- a/tactics/extraargs.ml4 +++ b/tactics/extraargs.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Pp open Pcoq open Genarg diff --git a/tactics/extraargs.mli b/tactics/extraargs.mli index 3421ded92..ffa1bd747 100644 --- a/tactics/extraargs.mli +++ b/tactics/extraargs.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Tacexpr open Term open Names diff --git a/tactics/extratactics.ml4 b/tactics/extratactics.ml4 index 8a68c9f20..a1c1da177 100644 --- a/tactics/extratactics.ml4 +++ b/tactics/extratactics.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Pp open Pcoq open Genarg diff --git a/tactics/extratactics.mli b/tactics/extratactics.mli index 259fe8814..f2f13fe11 100644 --- a/tactics/extratactics.mli +++ b/tactics/extratactics.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Proof_type val h_discrHyp : Names.identifier -> tactic diff --git a/tactics/hiddentac.ml b/tactics/hiddentac.ml index 4fed5d27c..da2b49557 100644 --- a/tactics/hiddentac.ml +++ b/tactics/hiddentac.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Term open Proof_type open Tacmach diff --git a/tactics/hiddentac.mli b/tactics/hiddentac.mli index dae0281bd..120d42abf 100644 --- a/tactics/hiddentac.mli +++ b/tactics/hiddentac.mli @@ -7,8 +7,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Util open Term diff --git a/tactics/hipattern.ml4 b/tactics/hipattern.ml4 index b6112c34f..b20383969 100644 --- a/tactics/hipattern.ml4 +++ b/tactics/hipattern.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma parsing/q_constr.cmo" i*) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/hipattern.mli b/tactics/hipattern.mli index 40ad0da9b..3fa8596f9 100644 --- a/tactics/hipattern.mli +++ b/tactics/hipattern.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/tactics/inv.ml b/tactics/inv.ml index 46ca8161c..3130c1ca9 100644 --- a/tactics/inv.ml +++ b/tactics/inv.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/inv.mli b/tactics/inv.mli index a7780206b..b038e4f0e 100644 --- a/tactics/inv.mli +++ b/tactics/inv.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/tactics/leminv.ml b/tactics/leminv.ml index 395a7c206..5c22bfd89 100644 --- a/tactics/leminv.ml +++ b/tactics/leminv.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/nbtermdn.ml b/tactics/nbtermdn.ml index 7d6e1c4c9..67b396dda 100644 --- a/tactics/nbtermdn.ml +++ b/tactics/nbtermdn.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Term diff --git a/tactics/nbtermdn.mli b/tactics/nbtermdn.mli index 3f866d5da..5d80d847e 100644 --- a/tactics/nbtermdn.mli +++ b/tactics/nbtermdn.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Pattern open Libnames diff --git a/tactics/refine.ml b/tactics/refine.ml index cb6cb961f..484954bcc 100644 --- a/tactics/refine.ml +++ b/tactics/refine.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* JCF -- 6 janvier 1998 EXPERIMENTAL *) (* diff --git a/tactics/refine.mli b/tactics/refine.mli index c9a4598e5..ef369a857 100644 --- a/tactics/refine.mli +++ b/tactics/refine.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Tacmach val refine : Evd.open_constr -> tactic diff --git a/tactics/rewrite.ml4 b/tactics/rewrite.ml4 index 1af2d3398..fd34d70f9 100644 --- a/tactics/rewrite.ml4 +++ b/tactics/rewrite.ml4 @@ -9,8 +9,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id: rewrite.ml4 11981 2009-03-16 08:18:53Z herbelin $ *) - open Pp open Util open Names diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml index 6e3957ac0..86bd7cbee 100644 --- a/tactics/tacinterp.ml +++ b/tactics/tacinterp.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Constrintern open Closure open RedFlags diff --git a/tactics/tacinterp.mli b/tactics/tacinterp.mli index 771d28fba..7c731e2b9 100644 --- a/tactics/tacinterp.mli +++ b/tactics/tacinterp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/tactics/tactic_option.ml b/tactics/tactic_option.ml index 8e5124c41..ff3abd1d2 100644 --- a/tactics/tactic_option.ml +++ b/tactics/tactic_option.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: subtac.ml 12623 2010-01-04 17:50:38Z letouzey $ *) - open Libobject open Proof_type open Pp diff --git a/tactics/tactic_option.mli b/tactics/tactic_option.mli index 208a76aef..d74bb0ebb 100644 --- a/tactics/tactic_option.mli +++ b/tactics/tactic_option.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: subtac.ml 12623 2010-01-04 17:50:38Z letouzey $ *) - open Proof_type open Tacexpr open Vernacexpr diff --git a/tactics/tacticals.ml b/tactics/tacticals.ml index 045f70c61..1ff67bffe 100644 --- a/tactics/tacticals.ml +++ b/tactics/tacticals.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/tacticals.mli b/tactics/tacticals.mli index c357451a2..e67e11227 100644 --- a/tactics/tacticals.mli +++ b/tactics/tacticals.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util open Names diff --git a/tactics/tactics.ml b/tactics/tactics.ml index e6201aad9..21a9ee258 100644 --- a/tactics/tactics.ml +++ b/tactics/tactics.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/tactics/tactics.mli b/tactics/tactics.mli index 2d7c07402..8a413e137 100644 --- a/tactics/tactics.mli +++ b/tactics/tactics.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/tactics/tauto.ml4 b/tactics/tauto.ml4 index 60baa017c..2bb225c66 100644 --- a/tactics/tauto.ml4 +++ b/tactics/tauto.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(*i $Id$ i*) - open Term open Hipattern open Names diff --git a/tactics/termdn.ml b/tactics/termdn.ml index 7b6d3ea76..fe5dc572d 100644 --- a/tactics/termdn.ml +++ b/tactics/termdn.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Names open Nameops diff --git a/tactics/termdn.mli b/tactics/termdn.mli index 973cc0e5b..ed3a928ab 100644 --- a/tactics/termdn.mli +++ b/tactics/termdn.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Term open Pattern open Libnames diff --git a/test-suite/bugs/closed/shouldsucceed/1507.v b/test-suite/bugs/closed/shouldsucceed/1507.v index f1872a2bb..f2ab91003 100644 --- a/test-suite/bugs/closed/shouldsucceed/1507.v +++ b/test-suite/bugs/closed/shouldsucceed/1507.v @@ -2,7 +2,6 @@ Implementing reals a la Stolzenberg Danko Ilik, March 2007 - svn revision: $Id$ XField.v -- (unfinished) axiomatisation of the theories of real and rational intervals. diff --git a/test-suite/misc/berardi_test.v b/test-suite/misc/berardi_test.v index 5b2f5063b..b32456a9e 100644 --- a/test-suite/misc/berardi_test.v +++ b/test-suite/misc/berardi_test.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file formalizes Berardi's paradox which says that in the calculus of constructions, excluded middle (EM) and axiom of choice (AC) imply proof irrelevance (PI). diff --git a/test-suite/success/Field.v b/test-suite/success/Field.v index dd82036e7..e30ab04ec 100644 --- a/test-suite/success/Field.v +++ b/test-suite/success/Field.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (**** Tests of Field with real numbers ****) Require Import Reals RealField. diff --git a/test-suite/success/LegacyField.v b/test-suite/success/LegacyField.v index fada3bd54..dbc0c056b 100644 --- a/test-suite/success/LegacyField.v +++ b/test-suite/success/LegacyField.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: Field.v 7693 2005-12-21 23:50:17Z herbelin $ *) - (**** Tests of Field with real numbers ****) Require Import Reals LegacyRfield. diff --git a/test-suite/success/Tauto.v b/test-suite/success/Tauto.v index 42898b8d1..b9e51e6cf 100644 --- a/test-suite/success/Tauto.v +++ b/test-suite/success/Tauto.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (**** Tactics Tauto and Intuition ****) (**** Tauto: diff --git a/test-suite/typeclasses/NewSetoid.v b/test-suite/typeclasses/NewSetoid.v index 8ad038809..de492cc42 100644 --- a/test-suite/typeclasses/NewSetoid.v +++ b/test-suite/typeclasses/NewSetoid.v @@ -11,8 +11,6 @@ * Institution: LRI, CNRS UMR 8623 - UniversitÃcopyright Paris Sud * 91405 Orsay, France *) -(* $Id: FSetAVL_prog.v 616 2007-08-08 12:28:10Z msozeau $ *) - Require Import Coq.Program.Program. Set Implicit Arguments. diff --git a/theories/Arith/Arith.v b/theories/Arith/Arith.v index 18dbd27f9..0de9136fd 100644 --- a/theories/Arith/Arith.v +++ b/theories/Arith/Arith.v @@ -6,7 +6,5 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Arith_base. Require Export ArithRing. diff --git a/theories/Arith/Arith_base.v b/theories/Arith/Arith_base.v index 2d54f0e8d..9395fc56c 100644 --- a/theories/Arith/Arith_base.v +++ b/theories/Arith/Arith_base.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Le. Require Export Lt. Require Export Plus. diff --git a/theories/Arith/Between.v b/theories/Arith/Between.v index 208c25789..b4cdb3c82 100644 --- a/theories/Arith/Between.v +++ b/theories/Arith/Between.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Le. Require Import Lt. diff --git a/theories/Arith/Bool_nat.v b/theories/Arith/Bool_nat.v index 9fd59e103..d94a71c9e 100644 --- a/theories/Arith/Bool_nat.v +++ b/theories/Arith/Bool_nat.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Compare_dec. Require Export Peano_dec. Require Import Sumbool. diff --git a/theories/Arith/Compare.v b/theories/Arith/Compare.v index 0f2595b26..c401eb283 100644 --- a/theories/Arith/Compare.v +++ b/theories/Arith/Compare.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Equality is decidable on [nat] *) Open Local Scope nat_scope. diff --git a/theories/Arith/Compare_dec.v b/theories/Arith/Compare_dec.v index 38d1aef0e..635b72671 100644 --- a/theories/Arith/Compare_dec.v +++ b/theories/Arith/Compare_dec.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Le. Require Import Lt. Require Import Gt. diff --git a/theories/Arith/Div2.v b/theories/Arith/Div2.v index 999a64544..c717e9bf5 100644 --- a/theories/Arith/Div2.v +++ b/theories/Arith/Div2.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Lt. Require Import Plus. Require Import Compare_dec. diff --git a/theories/Arith/EqNat.v b/theories/Arith/EqNat.v index 312b76e97..7d5b36ae5 100644 --- a/theories/Arith/EqNat.v +++ b/theories/Arith/EqNat.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Equality on natural numbers *) Open Local Scope nat_scope. diff --git a/theories/Arith/Euclid.v b/theories/Arith/Euclid.v index f50dcc84d..f118eb85b 100644 --- a/theories/Arith/Euclid.v +++ b/theories/Arith/Euclid.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Mult. Require Import Compare_dec. Require Import Wf_nat. diff --git a/theories/Arith/Even.v b/theories/Arith/Even.v index eaa1bb2d6..fa4414146 100644 --- a/theories/Arith/Even.v +++ b/theories/Arith/Even.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Here we define the predicates [even] and [odd] by mutual induction and we prove the decidability and the exclusion of those predicates. The main results about parity are proved in the module Div2. *) diff --git a/theories/Arith/Factorial.v b/theories/Arith/Factorial.v index 8c5315624..58631a987 100644 --- a/theories/Arith/Factorial.v +++ b/theories/Arith/Factorial.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Plus. Require Import Mult. Require Import Lt. diff --git a/theories/Arith/Gt.v b/theories/Arith/Gt.v index 70169f52a..20aad5c05 100644 --- a/theories/Arith/Gt.v +++ b/theories/Arith/Gt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Theorems about [gt] in [nat]. [gt] is defined in [Init/Peano.v] as: << Definition gt (n m:nat) := m < n. diff --git a/theories/Arith/Le.v b/theories/Arith/Le.v index 6140eeb5a..edf1e34d5 100644 --- a/theories/Arith/Le.v +++ b/theories/Arith/Le.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Order on natural numbers. [le] is defined in [Init/Peano.v] as: << Inductive le (n:nat) : nat -> Prop := diff --git a/theories/Arith/Lt.v b/theories/Arith/Lt.v index af435e54b..12819940d 100644 --- a/theories/Arith/Lt.v +++ b/theories/Arith/Lt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Theorems about [lt] in nat. [lt] is defined in library [Init/Peano.v] as: << Definition lt (n m:nat) := S n <= m. diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v index b94cc2485..ffce72774 100644 --- a/theories/Arith/Max.v +++ b/theories/Arith/Max.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** THIS FILE IS DEPRECATED. Use [NPeano.Nat] instead. *) Require Export NPeano. diff --git a/theories/Arith/Min.v b/theories/Arith/Min.v index ba03a40bd..c980baf09 100644 --- a/theories/Arith/Min.v +++ b/theories/Arith/Min.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** THIS FILE IS DEPRECATED. Use [NPeano.Nat] instead. *) Require Export NPeano. diff --git a/theories/Arith/Minus.v b/theories/Arith/Minus.v index cd6c0a29e..490bf8e55 100644 --- a/theories/Arith/Minus.v +++ b/theories/Arith/Minus.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** [minus] (difference between two natural numbers) is defined in [Init/Peano.v] as: << Fixpoint minus (n m:nat) : nat := diff --git a/theories/Arith/Mult.v b/theories/Arith/Mult.v index 8346cae38..811068daf 100644 --- a/theories/Arith/Mult.v +++ b/theories/Arith/Mult.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Plus. Require Export Minus. Require Export Lt. diff --git a/theories/Arith/Peano_dec.v b/theories/Arith/Peano_dec.v index 42335f98b..d8b46c78f 100644 --- a/theories/Arith/Peano_dec.v +++ b/theories/Arith/Peano_dec.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Decidable. Open Local Scope nat_scope. diff --git a/theories/Arith/Plus.v b/theories/Arith/Plus.v index 9b7c62615..28613eecc 100644 --- a/theories/Arith/Plus.v +++ b/theories/Arith/Plus.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Properties of addition. [add] is defined in [Init/Peano.v] as: << Fixpoint plus (n m:nat) : nat := diff --git a/theories/Arith/Wf_nat.v b/theories/Arith/Wf_nat.v index 5bc5d2a58..c12a577f8 100644 --- a/theories/Arith/Wf_nat.v +++ b/theories/Arith/Wf_nat.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Well-founded relations and natural numbers *) Require Import Lt. diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v index 66ab6f1c8..a1ea2ebc8 100644 --- a/theories/Bool/Bool.v +++ b/theories/Bool/Bool.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** The type [bool] is defined in the prelude as [Inductive bool : Set := true : bool | false : bool] *) diff --git a/theories/Bool/BoolEq.v b/theories/Bool/BoolEq.v index 625cbd194..9a2e738eb 100644 --- a/theories/Bool/BoolEq.v +++ b/theories/Bool/BoolEq.v @@ -6,7 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) (* Cuihtlauac Alvarado - octobre 2000 *) (** Properties of a boolean equality *) diff --git a/theories/Bool/Bvector.v b/theories/Bool/Bvector.v index d9da08672..b41d65c39 100644 --- a/theories/Bool/Bvector.v +++ b/theories/Bool/Bvector.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Bit vectors. Contribution by Jean Duprat (ENS Lyon). *) Require Export Bool Sumbool. diff --git a/theories/Bool/DecBool.v b/theories/Bool/DecBool.v index 90f7ee662..799438d89 100644 --- a/theories/Bool/DecBool.v +++ b/theories/Bool/DecBool.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Definition ifdec (A B:Prop) (C:Type) (H:{A} + {B}) (x y:C) : C := diff --git a/theories/Bool/IfProp.v b/theories/Bool/IfProp.v index c2b5ed793..573916ddc 100644 --- a/theories/Bool/IfProp.v +++ b/theories/Bool/IfProp.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Bool. Inductive IfProp (A B:Prop) : bool -> Prop := diff --git a/theories/Bool/Sumbool.v b/theories/Bool/Sumbool.v index 06ab77cfb..a34c49175 100644 --- a/theories/Bool/Sumbool.v +++ b/theories/Bool/Sumbool.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Here are collected some results about the type sumbool (see INIT/Specif.v) [sumbool A B], which is written [{A}+{B}], is the informative disjunction "A or B", where A and B are logical propositions. diff --git a/theories/Bool/Zerob.v b/theories/Bool/Zerob.v index 5e9d4afa6..fde053026 100644 --- a/theories/Bool/Zerob.v +++ b/theories/Bool/Zerob.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Arith. Require Import Bool. diff --git a/theories/Classes/EquivDec.v b/theories/Classes/EquivDec.v index 0a35ef45e..75c51a8dd 100644 --- a/theories/Classes/EquivDec.v +++ b/theories/Classes/EquivDec.v @@ -12,8 +12,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - (** Export notations. *) Require Export Coq.Classes.Equivalence. diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v index d0f243474..d62bd0674 100644 --- a/theories/Classes/Equivalence.v +++ b/theories/Classes/Equivalence.v @@ -12,8 +12,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Require Import Coq.Program.Basics. Require Import Coq.Program.Tactics. diff --git a/theories/Classes/Init.v b/theories/Classes/Init.v index f6e51018a..df288add4 100644 --- a/theories/Classes/Init.v +++ b/theories/Classes/Init.v @@ -13,8 +13,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - (** Hints for the proof search: these combinators should be considered rigid. *) Require Import Coq.Program.Basics. diff --git a/theories/Classes/Morphisms.v b/theories/Classes/Morphisms.v index 4b827c244..2421c90d0 100644 --- a/theories/Classes/Morphisms.v +++ b/theories/Classes/Morphisms.v @@ -13,8 +13,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Require Import Coq.Program.Basics. Require Import Coq.Program.Tactics. Require Import Coq.Relations.Relation_Definitions. diff --git a/theories/Classes/RelationClasses.v b/theories/Classes/RelationClasses.v index a8193ef3c..4c39964a9 100644 --- a/theories/Classes/RelationClasses.v +++ b/theories/Classes/RelationClasses.v @@ -15,8 +15,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Require Export Coq.Classes.Init. Require Import Coq.Program.Basics. Require Import Coq.Program.Tactics. diff --git a/theories/Classes/SetoidClass.v b/theories/Classes/SetoidClass.v index c41c57698..36fe2b9a6 100644 --- a/theories/Classes/SetoidClass.v +++ b/theories/Classes/SetoidClass.v @@ -12,8 +12,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Set Implicit Arguments. Unset Strict Implicit. diff --git a/theories/Classes/SetoidDec.v b/theories/Classes/SetoidDec.v index 33b4350f8..ab2131185 100644 --- a/theories/Classes/SetoidDec.v +++ b/theories/Classes/SetoidDec.v @@ -13,8 +13,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Set Implicit Arguments. Unset Strict Implicit. diff --git a/theories/Classes/SetoidTactics.v b/theories/Classes/SetoidTactics.v index 669be8b0f..dbdff45f3 100644 --- a/theories/Classes/SetoidTactics.v +++ b/theories/Classes/SetoidTactics.v @@ -12,8 +12,6 @@ Institution: LRI, CNRS UMR 8623 - University Paris Sud *) -(* $Id$ *) - Require Import Coq.Classes.Morphisms Coq.Classes.Morphisms_Prop. Require Export Coq.Classes.RelationClasses Coq.Relations.Relation_Definitions. Require Import Coq.Classes.Equivalence Coq.Program.Basics. diff --git a/theories/FSets/FMapAVL.v b/theories/FSets/FMapAVL.v index c6252de9c..e0ddbe3ab 100644 --- a/theories/FSets/FMapAVL.v +++ b/theories/FSets/FMapAVL.v @@ -8,8 +8,6 @@ (* Finite map library. *) -(* $Id$ *) - (** * FMapAVL *) (** This module implements maps using AVL trees. diff --git a/theories/FSets/FMapFacts.v b/theories/FSets/FMapFacts.v index 4c59971cb..fd58ec10a 100644 --- a/theories/FSets/FMapFacts.v +++ b/theories/FSets/FMapFacts.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite maps library *) (** This functor derives additional facts from [FMapInterface.S]. These diff --git a/theories/FSets/FMapFullAVL.v b/theories/FSets/FMapFullAVL.v index afac5af8c..1facce290 100644 --- a/theories/FSets/FMapFullAVL.v +++ b/theories/FSets/FMapFullAVL.v @@ -8,8 +8,6 @@ (* Finite map library. *) -(* $Id$ *) - (** * FMapFullAVL This file contains some complements to [FMapAVL]. diff --git a/theories/FSets/FMapInterface.v b/theories/FSets/FMapInterface.v index e60cca9d9..252e67930 100644 --- a/theories/FSets/FMapInterface.v +++ b/theories/FSets/FMapInterface.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite map library *) (** This file proposes interfaces for finite maps *) diff --git a/theories/FSets/FMapList.v b/theories/FSets/FMapList.v index 56fc35d89..f15ab222c 100644 --- a/theories/FSets/FMapList.v +++ b/theories/FSets/FMapList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite map library *) (** This file proposes an implementation of the non-dependant interface diff --git a/theories/FSets/FMapPositive.v b/theories/FSets/FMapPositive.v index 56ad2ed11..e85cc283e 100644 --- a/theories/FSets/FMapPositive.v +++ b/theories/FSets/FMapPositive.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * FMapPositive : an implementation of FMapInterface for [positive] keys. *) Require Import Bool. diff --git a/theories/FSets/FMapWeakList.v b/theories/FSets/FMapWeakList.v index 38ed172b8..6c1e8ca89 100644 --- a/theories/FSets/FMapWeakList.v +++ b/theories/FSets/FMapWeakList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite map library *) (** This file proposes an implementation of the non-dependant interface diff --git a/theories/FSets/FMaps.v b/theories/FSets/FMaps.v index 6b1102406..19b25d95a 100644 --- a/theories/FSets/FMaps.v +++ b/theories/FSets/FMaps.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export OrderedType OrderedTypeEx OrderedTypeAlt. Require Export DecidableType DecidableTypeEx. diff --git a/theories/FSets/FSetAVL.v b/theories/FSets/FSetAVL.v index bc6c731f6..df627a14b 100644 --- a/theories/FSets/FSetAVL.v +++ b/theories/FSets/FSetAVL.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * FSetAVL : Implementation of FSetInterface via AVL trees *) (** This module implements finite sets using AVL trees. diff --git a/theories/FSets/FSetBridge.v b/theories/FSets/FSetBridge.v index 1b1bae352..8d6ca420b 100644 --- a/theories/FSets/FSetBridge.v +++ b/theories/FSets/FSetBridge.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This module implements bridges (as functors) from dependent diff --git a/theories/FSets/FSetDecide.v b/theories/FSets/FSetDecide.v index 89cdc932f..a87103232 100644 --- a/theories/FSets/FSetDecide.v +++ b/theories/FSets/FSetDecide.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (**************************************************************) (* FSetDecide.v *) (* *) diff --git a/theories/FSets/FSetEqProperties.v b/theories/FSets/FSetEqProperties.v index ec0c6a559..755bc7dd0 100644 --- a/theories/FSets/FSetEqProperties.v +++ b/theories/FSets/FSetEqProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This module proves many properties of finite sets that diff --git a/theories/FSets/FSetFacts.v b/theories/FSets/FSetFacts.v index b750edfc0..f473b3342 100644 --- a/theories/FSets/FSetFacts.v +++ b/theories/FSets/FSetFacts.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This functor derives additional facts from [FSetInterface.S]. These diff --git a/theories/FSets/FSetInterface.v b/theories/FSets/FSetInterface.v index 8aede5527..a23263890 100644 --- a/theories/FSets/FSetInterface.v +++ b/theories/FSets/FSetInterface.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite set library *) (** Set interfaces, inspired by the one of Ocaml. When compared with diff --git a/theories/FSets/FSetList.v b/theories/FSets/FSetList.v index f83259c44..1f36306c3 100644 --- a/theories/FSets/FSetList.v +++ b/theories/FSets/FSetList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This file proposes an implementation of the non-dependant diff --git a/theories/FSets/FSetProperties.v b/theories/FSets/FSetProperties.v index 84c26dacd..80da1c5d8 100644 --- a/theories/FSets/FSetProperties.v +++ b/theories/FSets/FSetProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This functor derives additional properties from [FSetInterface.S]. diff --git a/theories/FSets/FSetToFiniteSet.v b/theories/FSets/FSetToFiniteSet.v index 01138270e..3ac5d9e4a 100644 --- a/theories/FSets/FSetToFiniteSet.v +++ b/theories/FSets/FSetToFiniteSet.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library : conversion to old [Finite_sets] *) Require Import Ensembles Finite_sets. diff --git a/theories/FSets/FSetWeakList.v b/theories/FSets/FSetWeakList.v index 711cbd9a6..2ea32e97c 100644 --- a/theories/FSets/FSetWeakList.v +++ b/theories/FSets/FSetWeakList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This file proposes an implementation of the non-dependant diff --git a/theories/FSets/FSets.v b/theories/FSets/FSets.v index eaa8f4034..9a7294119 100644 --- a/theories/FSets/FSets.v +++ b/theories/FSets/FSets.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export OrderedType. Require Export OrderedTypeEx. Require Export OrderedTypeAlt. diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v index 092fce996..782ff6ca9 100644 --- a/theories/Init/Datatypes.v +++ b/theories/Init/Datatypes.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import Notations. diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 4fca1d1db..14832e0b7 100644 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import Notations. diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v index 1333f3545..ff6a18e14 100644 --- a/theories/Init/Logic_Type.v +++ b/theories/Init/Logic_Type.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This module defines type constructors for types in [Type] ([Datatypes.v] and [Logic.v] defined them for types in [Set]) *) diff --git a/theories/Init/Notations.v b/theories/Init/Notations.v index 0c628298d..9bf921b22 100644 --- a/theories/Init/Notations.v +++ b/theories/Init/Notations.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** These are the notations whose level and associativity are imposed by Coq *) (** Notations for propositional connectives *) diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v index 8779f2b45..045210d0a 100644 --- a/theories/Init/Peano.v +++ b/theories/Init/Peano.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** The type [nat] of Peano natural numbers (built from [O] and [S]) is defined in [Datatypes.v] *) diff --git a/theories/Init/Prelude.v b/theories/Init/Prelude.v index 45b949716..c8d809fd4 100644 --- a/theories/Init/Prelude.v +++ b/theories/Init/Prelude.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Notations. Require Export Logic. Require Export Datatypes. diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v index 7141f26cb..6ff820299 100644 --- a/theories/Init/Specif.v +++ b/theories/Init/Specif.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Basic specifications : sets that may contain logical information *) Set Implicit Arguments. diff --git a/theories/Init/Tactics.v b/theories/Init/Tactics.v index 6ccf8a022..66f90e18f 100644 --- a/theories/Init/Tactics.v +++ b/theories/Init/Tactics.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Notations. Require Import Logic. Require Import Specif. diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v index 3209860f3..0a1a0f9b8 100644 --- a/theories/Init/Wf.v +++ b/theories/Init/Wf.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** * This module proves the validity of - well-founded recursion (also known as course of values) - well-founded induction diff --git a/theories/Lists/List.v b/theories/Lists/List.v index 766456fff..d1e3f90b3 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Le Gt Minus Bool. Set Implicit Arguments. diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v index e6c3a435b..0ed3bbbb7 100644 --- a/theories/Lists/ListSet.v +++ b/theories/Lists/ListSet.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** A Library for finite sets, implemented as lists *) (** List is loaded, but not exported. diff --git a/theories/Lists/ListTactics.v b/theories/Lists/ListTactics.v index 0a21a9e27..3a743dd47 100644 --- a/theories/Lists/ListTactics.v +++ b/theories/Lists/ListTactics.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinPos. Require Import List. diff --git a/theories/Lists/SetoidList.v b/theories/Lists/SetoidList.v index d42e71e55..88ccdb126 100644 --- a/theories/Lists/SetoidList.v +++ b/theories/Lists/SetoidList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export List. Require Export Sorting. Require Export Setoid Basics Morphisms. diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v index 3fa053b7f..39a2968f7 100644 --- a/theories/Lists/Streams.v +++ b/theories/Lists/Streams.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. (** Streams *) diff --git a/theories/Lists/TheoryList.v b/theories/Lists/TheoryList.v index 7ed9c519b..2d75f065f 100644 --- a/theories/Lists/TheoryList.v +++ b/theories/Lists/TheoryList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Some programs and results about lists following CAML Manual *) Require Export List. diff --git a/theories/Logic/Berardi.v b/theories/Logic/Berardi.v index 5b2f5063b..b32456a9e 100644 --- a/theories/Logic/Berardi.v +++ b/theories/Logic/Berardi.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file formalizes Berardi's paradox which says that in the calculus of constructions, excluded middle (EM) and axiom of choice (AC) imply proof irrelevance (PI). diff --git a/theories/Logic/ChoiceFacts.v b/theories/Logic/ChoiceFacts.v index b2c4a049d..903081ce6 100644 --- a/theories/Logic/ChoiceFacts.v +++ b/theories/Logic/ChoiceFacts.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: ChoiceFacts.v 12363 2009-09-28 15:04:07Z letouzey $ i*) - (** Some facts and definitions concerning choice and description in intuitionistic logic. diff --git a/theories/Logic/Classical.v b/theories/Logic/Classical.v index 1c2b97ce7..4a01f3fae 100644 --- a/theories/Logic/Classical.v +++ b/theories/Logic/Classical.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Classical Logic *) Require Export Classical_Prop. diff --git a/theories/Logic/ClassicalChoice.v b/theories/Logic/ClassicalChoice.v index b0301994b..92e48e6a9 100644 --- a/theories/Logic/ClassicalChoice.v +++ b/theories/Logic/ClassicalChoice.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides classical logic and functional choice; this especially provides both indefinite descriptions and choice functions but this is weaker than providing epsilon operator and classical logic diff --git a/theories/Logic/ClassicalDescription.v b/theories/Logic/ClassicalDescription.v index 2b9df6d97..a5d1babaa 100644 --- a/theories/Logic/ClassicalDescription.v +++ b/theories/Logic/ClassicalDescription.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides classical logic and definite description, which is equivalent to providing classical logic and Church's iota operator *) diff --git a/theories/Logic/ClassicalEpsilon.v b/theories/Logic/ClassicalEpsilon.v index cee55dc81..7de6ddab6 100644 --- a/theories/Logic/ClassicalEpsilon.v +++ b/theories/Logic/ClassicalEpsilon.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides classical logic and indefinite description under the form of Hilbert's epsilon operator *) diff --git a/theories/Logic/ClassicalFacts.v b/theories/Logic/ClassicalFacts.v index b22a3a874..a271c05bc 100644 --- a/theories/Logic/ClassicalFacts.v +++ b/theories/Logic/ClassicalFacts.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Some facts and definitions about classical logic Table of contents: diff --git a/theories/Logic/ClassicalUniqueChoice.v b/theories/Logic/ClassicalUniqueChoice.v index 4a7bd2ccc..67b853be9 100644 --- a/theories/Logic/ClassicalUniqueChoice.v +++ b/theories/Logic/ClassicalUniqueChoice.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides classical logic and unique choice; this is weaker than providing iota operator and classical logic as the definite descriptions provided by the axiom of unique choice can diff --git a/theories/Logic/Classical_Pred_Set.v b/theories/Logic/Classical_Pred_Set.v index 0b0c329be..afbb5e6df 100644 --- a/theories/Logic/Classical_Pred_Set.v +++ b/theories/Logic/Classical_Pred_Set.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file is obsolete, use Classical_Pred_Type.v via Classical.v instead *) diff --git a/theories/Logic/Classical_Pred_Type.v b/theories/Logic/Classical_Pred_Type.v index b30308af5..45c487cf7 100644 --- a/theories/Logic/Classical_Pred_Type.v +++ b/theories/Logic/Classical_Pred_Type.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Classical Predicate Logic on Type *) Require Import Classical_Prop. diff --git a/theories/Logic/Classical_Prop.v b/theories/Logic/Classical_Prop.v index df732959f..ee6dd96f2 100644 --- a/theories/Logic/Classical_Prop.v +++ b/theories/Logic/Classical_Prop.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Classical Propositional Logic *) Require Import ClassicalFacts. diff --git a/theories/Logic/Classical_Type.v b/theories/Logic/Classical_Type.v index 3b91afd02..b3053fa1d 100644 --- a/theories/Logic/Classical_Type.v +++ b/theories/Logic/Classical_Type.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file is obsolete, use Classical.v instead *) (** Classical Logic for Type *) diff --git a/theories/Logic/ConstructiveEpsilon.v b/theories/Logic/ConstructiveEpsilon.v index 6d22b1a9e..8077cabf7 100644 --- a/theories/Logic/ConstructiveEpsilon.v +++ b/theories/Logic/ConstructiveEpsilon.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This module proves the constructive description schema, which infers the sigma-existence (i.e., [Set]-existence) of a witness to a predicate from the regular existence (i.e., [Prop]-existence). One diff --git a/theories/Logic/Decidable.v b/theories/Logic/Decidable.v index c6d32d9be..75441584d 100644 --- a/theories/Logic/Decidable.v +++ b/theories/Logic/Decidable.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Properties of decidable propositions *) Definition decidable (P:Prop) := P \/ ~ P. diff --git a/theories/Logic/Description.v b/theories/Logic/Description.v index a8a56ae74..dd1d56b31 100644 --- a/theories/Logic/Description.v +++ b/theories/Logic/Description.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides a constructive form of definite description; it allows to build functions from the proof of their existence in any context; this is weaker than Church's iota operator *) diff --git a/theories/Logic/Diaconescu.v b/theories/Logic/Diaconescu.v index 18f3181b6..b513bdf73 100644 --- a/theories/Logic/Diaconescu.v +++ b/theories/Logic/Diaconescu.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Diaconescu showed that the Axiom of Choice entails Excluded-Middle in topoi [Diaconescu75]. Lacas and Werner adapted the proof to show that the axiom of choice in equivalence classes entails diff --git a/theories/Logic/Epsilon.v b/theories/Logic/Epsilon.v index d433be944..7de0aa7fc 100644 --- a/theories/Logic/Epsilon.v +++ b/theories/Logic/Epsilon.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides indefinite description under the form of Hilbert's epsilon operator; it does not assume classical logic. *) diff --git a/theories/Logic/Eqdep.v b/theories/Logic/Eqdep.v index 5c6b4e89f..14ab70b67 100644 --- a/theories/Logic/Eqdep.v +++ b/theories/Logic/Eqdep.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file axiomatizes the invariance by substitution of reflexive equality proofs [[Streicher93]] and exports its consequences, such as the injectivity of the projection of the dependent pair. diff --git a/theories/Logic/EqdepFacts.v b/theories/Logic/EqdepFacts.v index 4689fb46c..9c20905c7 100644 --- a/theories/Logic/EqdepFacts.v +++ b/theories/Logic/EqdepFacts.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file defines dependent equality and shows its equivalence with equality on dependent pairs (inhabiting sigma-types). It derives the consequence of axiomatizing the invariance by substitution of diff --git a/theories/Logic/Eqdep_dec.v b/theories/Logic/Eqdep_dec.v index c7cb9b0d4..d4d05fe1a 100644 --- a/theories/Logic/Eqdep_dec.v +++ b/theories/Logic/Eqdep_dec.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** We prove that there is only one proof of [x=x], i.e [refl_equal x]. This holds if the equality upon the set of [x] is decidable. A corollary of this theorem is the equality of the right projections diff --git a/theories/Logic/FunctionalExtensionality.v b/theories/Logic/FunctionalExtensionality.v index bf29c63dd..5d6a4f7d6 100644 --- a/theories/Logic/FunctionalExtensionality.v +++ b/theories/Logic/FunctionalExtensionality.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This module states the axiom of (dependent) functional extensionality and (dependent) eta-expansion. It introduces a tactic [extensionality] to apply the axiom of extensionality to an equality goal. *) diff --git a/theories/Logic/IndefiniteDescription.v b/theories/Logic/IndefiniteDescription.v index 3651c1b2f..94922525b 100644 --- a/theories/Logic/IndefiniteDescription.v +++ b/theories/Logic/IndefiniteDescription.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file provides a constructive form of indefinite description that allows to build choice functions; this is weaker than Hilbert's epsilon operator (which implies weakly classical properties) but diff --git a/theories/Logic/JMeq.v b/theories/Logic/JMeq.v index fc4555a4a..f17e403ed 100644 --- a/theories/Logic/JMeq.v +++ b/theories/Logic/JMeq.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** John Major's Equality as proposed by Conor McBride Reference: diff --git a/theories/Logic/RelationalChoice.v b/theories/Logic/RelationalChoice.v index 49fa12224..9313e1073 100644 --- a/theories/Logic/RelationalChoice.v +++ b/theories/Logic/RelationalChoice.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file axiomatizes the relational form of the axiom of choice *) Axiom relational_choice : diff --git a/theories/MSets/MSetAVL.v b/theories/MSets/MSetAVL.v index f79f8d0b2..0d24e0339 100644 --- a/theories/MSets/MSetAVL.v +++ b/theories/MSets/MSetAVL.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * MSetAVL : Implementation of MSetInterface via AVL trees *) (** This module implements finite sets using AVL trees. diff --git a/theories/MSets/MSetDecide.v b/theories/MSets/MSetDecide.v index 884ed4235..1161739ed 100644 --- a/theories/MSets/MSetDecide.v +++ b/theories/MSets/MSetDecide.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (**************************************************************) (* MSetDecide.v *) (* *) diff --git a/theories/MSets/MSetEqProperties.v b/theories/MSets/MSetEqProperties.v index fe6c3c79c..2e7da404e 100644 --- a/theories/MSets/MSetEqProperties.v +++ b/theories/MSets/MSetEqProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This module proves many properties of finite sets that diff --git a/theories/MSets/MSetFacts.v b/theories/MSets/MSetFacts.v index 84f6a1705..b61bf3fe7 100644 --- a/theories/MSets/MSetFacts.v +++ b/theories/MSets/MSetFacts.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This functor derives additional facts from [MSetInterface.S]. These diff --git a/theories/MSets/MSetInterface.v b/theories/MSets/MSetInterface.v index 10776a590..7dc3c96a8 100644 --- a/theories/MSets/MSetInterface.v +++ b/theories/MSets/MSetInterface.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite set library *) (** Set interfaces, inspired by the one of Ocaml. When compared with diff --git a/theories/MSets/MSetList.v b/theories/MSets/MSetList.v index 0414e6eda..b73af8f1a 100644 --- a/theories/MSets/MSetList.v +++ b/theories/MSets/MSetList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This file proposes an implementation of the non-dependant diff --git a/theories/MSets/MSetProperties.v b/theories/MSets/MSetProperties.v index a9ba0a823..14fe097a9 100644 --- a/theories/MSets/MSetProperties.v +++ b/theories/MSets/MSetProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This functor derives additional properties from [MSetInterface.S]. diff --git a/theories/MSets/MSetToFiniteSet.v b/theories/MSets/MSetToFiniteSet.v index f0b964cf2..e8087bc57 100644 --- a/theories/MSets/MSetToFiniteSet.v +++ b/theories/MSets/MSetToFiniteSet.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library : conversion to old [Finite_sets] *) Require Import Ensembles Finite_sets. diff --git a/theories/MSets/MSetWeakList.v b/theories/MSets/MSetWeakList.v index 6b9c17079..8239ecef8 100644 --- a/theories/MSets/MSetWeakList.v +++ b/theories/MSets/MSetWeakList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * Finite sets library *) (** This file proposes an implementation of the non-dependant diff --git a/theories/MSets/MSets.v b/theories/MSets/MSets.v index 558b09562..a4b9efc3b 100644 --- a/theories/MSets/MSets.v +++ b/theories/MSets/MSets.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export Orders. Require Export OrdersEx. Require Export OrdersAlt. diff --git a/theories/NArith/BinNat.v b/theories/NArith/BinNat.v index b289380fd..6b668df60 100644 --- a/theories/NArith/BinNat.v +++ b/theories/NArith/BinNat.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinPos. Unset Boxed Definitions. diff --git a/theories/NArith/BinPos.v b/theories/NArith/BinPos.v index a5f99cc66..a7b2336c8 100644 --- a/theories/NArith/BinPos.v +++ b/theories/NArith/BinPos.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Unset Boxed Definitions. Declare ML Module "z_syntax_plugin". diff --git a/theories/NArith/NArith.v b/theories/NArith/NArith.v index 009e64fd0..7282fc758 100644 --- a/theories/NArith/NArith.v +++ b/theories/NArith/NArith.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Library for binary natural numbers *) Require Export BinPos. diff --git a/theories/NArith/Ndec.v b/theories/NArith/Ndec.v index 9540aace7..c217ada11 100644 --- a/theories/NArith/Ndec.v +++ b/theories/NArith/Ndec.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Bool. Require Import Sumbool. Require Import Arith. diff --git a/theories/NArith/Ndigits.v b/theories/NArith/Ndigits.v index b699b7428..a79cfac3d 100644 --- a/theories/NArith/Ndigits.v +++ b/theories/NArith/Ndigits.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Bool Setoid Bvector BinPos BinNat. (** Operation over bits of a [N] number. *) diff --git a/theories/NArith/Ndist.v b/theories/NArith/Ndist.v index 92559ff67..dc37fa6c2 100644 --- a/theories/NArith/Ndist.v +++ b/theories/NArith/Ndist.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Arith. Require Import Min. Require Import BinPos. diff --git a/theories/NArith/Nnat.v b/theories/NArith/Nnat.v index 0016d035f..feabd3b16 100644 --- a/theories/NArith/Nnat.v +++ b/theories/NArith/Nnat.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Arith_base. Require Import Compare_dec. Require Import Sumbool. diff --git a/theories/NArith/Pnat.v b/theories/NArith/Pnat.v index 0891dea21..fea12a1d4 100644 --- a/theories/NArith/Pnat.v +++ b/theories/NArith/Pnat.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinPos. (**********************************************************************) diff --git a/theories/Numbers/BigNumPrelude.v b/theories/Numbers/BigNumPrelude.v index 08da68444..f11fb67b1 100644 --- a/theories/Numbers/BigNumPrelude.v +++ b/theories/Numbers/BigNumPrelude.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - (** * BigNumPrelude *) (** Auxillary functions & theorems used for arbitrary precision efficient diff --git a/theories/Numbers/Cyclic/Abstract/CyclicAxioms.v b/theories/Numbers/Cyclic/Abstract/CyclicAxioms.v index af30b0175..0403722cb 100644 --- a/theories/Numbers/Cyclic/Abstract/CyclicAxioms.v +++ b/theories/Numbers/Cyclic/Abstract/CyclicAxioms.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(* $Id$ *) - (** * Signature and specification of a bounded integer structure *) (** This file specifies how to represent [Z/nZ] when [n=2^d], diff --git a/theories/Numbers/Cyclic/Abstract/NZCyclic.v b/theories/Numbers/Cyclic/Abstract/NZCyclic.v index b68e89560..0796d9f49 100644 --- a/theories/Numbers/Cyclic/Abstract/NZCyclic.v +++ b/theories/Numbers/Cyclic/Abstract/NZCyclic.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NZAxioms. Require Import BigNumPrelude. Require Import DoubleType. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleAdd.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleAdd.v index aa798e1c7..81b2c9403 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleAdd.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleAdd.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleBase.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleBase.v index 23c62740c..bf18c1753 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleBase.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleBase.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleCyclic.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleCyclic.v index 49a4f950a..a640aaf7f 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleCyclic.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleCyclic.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleDiv.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleDiv.v index 1ce1e81b0..ae806dd5e 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleDiv.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleDiv.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleDivn1.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleDivn1.v index 136f96c04..1c4247231 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleDivn1.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleDivn1.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleLift.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleLift.v index 3405b6f4d..1395caa33 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleLift.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleLift.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleMul.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleMul.v index 6a2a34449..8b978172c 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleMul.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleMul.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleSqrt.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleSqrt.v index e2c623201..81df55bd4 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleSqrt.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleSqrt.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleSub.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleSub.v index a7e556713..a5610fe78 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleSub.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleSub.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/DoubleCyclic/DoubleType.v b/theories/Numbers/Cyclic/DoubleCyclic/DoubleType.v index 88cbb484f..da75219a5 100644 --- a/theories/Numbers/Cyclic/DoubleCyclic/DoubleType.v +++ b/theories/Numbers/Cyclic/DoubleCyclic/DoubleType.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Set Implicit Arguments. Require Import ZArith. diff --git a/theories/Numbers/Cyclic/Int31/Cyclic31.v b/theories/Numbers/Cyclic/Int31/Cyclic31.v index e2e5b563f..ca73a9f00 100644 --- a/theories/Numbers/Cyclic/Int31/Cyclic31.v +++ b/theories/Numbers/Cyclic/Int31/Cyclic31.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** * Int31 numbers defines indeed a cyclic structure : Z/(2^31)Z *) (** diff --git a/theories/Numbers/Cyclic/Int31/Int31.v b/theories/Numbers/Cyclic/Int31/Int31.v index cc224254f..9b4c25e2c 100644 --- a/theories/Numbers/Cyclic/Int31/Int31.v +++ b/theories/Numbers/Cyclic/Int31/Int31.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NaryFunctions. Require Import Wf_nat. Require Export ZArith. diff --git a/theories/Numbers/Cyclic/Int31/Ring31.v b/theories/Numbers/Cyclic/Int31/Ring31.v index a9c499fb9..01002656d 100644 --- a/theories/Numbers/Cyclic/Int31/Ring31.v +++ b/theories/Numbers/Cyclic/Int31/Ring31.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** * Int31 numbers defines Z/(2^31)Z, and can hence be equipped with a ring structure and a ring tactic *) diff --git a/theories/Numbers/Cyclic/ZModulo/ZModulo.v b/theories/Numbers/Cyclic/ZModulo/ZModulo.v index da0be5e2a..a2ee248ab 100644 --- a/theories/Numbers/Cyclic/ZModulo/ZModulo.v +++ b/theories/Numbers/Cyclic/ZModulo/ZModulo.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** * Type [Z] viewed modulo a particular constant corresponds to [Z/nZ] as defined abstractly in CyclicAxioms. *) diff --git a/theories/Numbers/Integer/Abstract/ZAdd.v b/theories/Numbers/Integer/Abstract/ZAdd.v index 5663408d1..123c40428 100644 --- a/theories/Numbers/Integer/Abstract/ZAdd.v +++ b/theories/Numbers/Integer/Abstract/ZAdd.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZBase. Module ZAddPropFunct (Import Z : ZAxiomsSig'). diff --git a/theories/Numbers/Integer/Abstract/ZAddOrder.v b/theories/Numbers/Integer/Abstract/ZAddOrder.v index de12993f8..adc843264 100644 --- a/theories/Numbers/Integer/Abstract/ZAddOrder.v +++ b/theories/Numbers/Integer/Abstract/ZAddOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZLt. Module ZAddOrderPropFunct (Import Z : ZAxiomsSig'). diff --git a/theories/Numbers/Integer/Abstract/ZAxioms.v b/theories/Numbers/Integer/Abstract/ZAxioms.v index 9158a214d..46f7810ac 100644 --- a/theories/Numbers/Integer/Abstract/ZAxioms.v +++ b/theories/Numbers/Integer/Abstract/ZAxioms.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NZAxioms. Set Implicit Arguments. diff --git a/theories/Numbers/Integer/Abstract/ZBase.v b/theories/Numbers/Integer/Abstract/ZBase.v index 44bb02ecc..ca288e6b2 100644 --- a/theories/Numbers/Integer/Abstract/ZBase.v +++ b/theories/Numbers/Integer/Abstract/ZBase.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export Decidable. Require Export ZAxioms. Require Import NZProperties. diff --git a/theories/Numbers/Integer/Abstract/ZLt.v b/theories/Numbers/Integer/Abstract/ZLt.v index 849bf6b40..fdb7c77f6 100644 --- a/theories/Numbers/Integer/Abstract/ZLt.v +++ b/theories/Numbers/Integer/Abstract/ZLt.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZMul. Module ZOrderPropFunct (Import Z : ZAxiomsSig'). diff --git a/theories/Numbers/Integer/Abstract/ZMul.v b/theories/Numbers/Integer/Abstract/ZMul.v index 84d840ad2..4a87a54c8 100644 --- a/theories/Numbers/Integer/Abstract/ZMul.v +++ b/theories/Numbers/Integer/Abstract/ZMul.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZAdd. Module ZMulPropFunct (Import Z : ZAxiomsSig'). diff --git a/theories/Numbers/Integer/Abstract/ZMulOrder.v b/theories/Numbers/Integer/Abstract/ZMulOrder.v index 99be58ebd..1952f4e2a 100644 --- a/theories/Numbers/Integer/Abstract/ZMulOrder.v +++ b/theories/Numbers/Integer/Abstract/ZMulOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZAddOrder. Module Type ZMulOrderPropFunct (Import Z : ZAxiomsSig'). diff --git a/theories/Numbers/Integer/Abstract/ZProperties.v b/theories/Numbers/Integer/Abstract/ZProperties.v index 45662d3b6..76451da33 100644 --- a/theories/Numbers/Integer/Abstract/ZProperties.v +++ b/theories/Numbers/Integer/Abstract/ZProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZAxioms ZMaxMin ZSgnAbs. (** This functor summarizes all known facts about Z. diff --git a/theories/Numbers/Integer/BigZ/BigZ.v b/theories/Numbers/Integer/BigZ/BigZ.v index aa62ae76b..c0b8074b6 100644 --- a/theories/Numbers/Integer/BigZ/BigZ.v +++ b/theories/Numbers/Integer/BigZ/BigZ.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export BigN. Require Import ZProperties ZDivFloor ZSig ZSigZAxioms ZMake. diff --git a/theories/Numbers/Integer/BigZ/ZMake.v b/theories/Numbers/Integer/BigZ/ZMake.v index 3196f11ea..41b1d6e69 100644 --- a/theories/Numbers/Integer/BigZ/ZMake.v +++ b/theories/Numbers/Integer/BigZ/ZMake.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith. Require Import BigNumPrelude. Require Import NSig. diff --git a/theories/Numbers/Integer/Binary/ZBinary.v b/theories/Numbers/Integer/Binary/ZBinary.v index bc1dadcd9..aa857f3ca 100644 --- a/theories/Numbers/Integer/Binary/ZBinary.v +++ b/theories/Numbers/Integer/Binary/ZBinary.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZAxioms ZProperties. Require Import BinInt Zcompare Zorder ZArith_dec Zbool. diff --git a/theories/Numbers/Integer/NatPairs/ZNatPairs.v b/theories/Numbers/Integer/NatPairs/ZNatPairs.v index 8b5624cdf..cafcc549e 100644 --- a/theories/Numbers/Integer/NatPairs/ZNatPairs.v +++ b/theories/Numbers/Integer/NatPairs/ZNatPairs.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NProperties. (* The most complete file for N *) Require Export ZProperties. (* The most complete file for Z *) Require Export Ring. diff --git a/theories/Numbers/Integer/SpecViaZ/ZSig.v b/theories/Numbers/Integer/SpecViaZ/ZSig.v index ffa91706f..ab12e584b 100644 --- a/theories/Numbers/Integer/SpecViaZ/ZSig.v +++ b/theories/Numbers/Integer/SpecViaZ/ZSig.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith Znumtheory. Open Scope Z_scope. diff --git a/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v b/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v index bcecb6a8a..2c4797969 100644 --- a/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v +++ b/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith ZAxioms ZDivFloor ZSig. (** * The interface [ZSig.ZType] implies the interface [ZAxiomsSig] diff --git a/theories/Numbers/NaryFunctions.v b/theories/Numbers/NaryFunctions.v index 417463eba..121b33b00 100644 --- a/theories/Numbers/NaryFunctions.v +++ b/theories/Numbers/NaryFunctions.v @@ -8,8 +8,6 @@ (* Pierre Letouzey, Jerome Vouillon, PPS, Paris 7, 2008 *) (************************************************************************) -(*i $Id$ i*) - Local Open Scope type_scope. Require Import List. diff --git a/theories/Numbers/NatInt/NZAdd.v b/theories/Numbers/NatInt/NZAdd.v index 9535cfdb4..37a174c48 100644 --- a/theories/Numbers/NatInt/NZAdd.v +++ b/theories/Numbers/NatInt/NZAdd.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms NZBase. Module Type NZAddPropSig diff --git a/theories/Numbers/NatInt/NZAddOrder.v b/theories/Numbers/NatInt/NZAddOrder.v index 97c122029..66e9c6ceb 100644 --- a/theories/Numbers/NatInt/NZAddOrder.v +++ b/theories/Numbers/NatInt/NZAddOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms NZBase NZMul NZOrder. Module Type NZAddOrderPropSig (Import NZ : NZOrdAxiomsSig'). diff --git a/theories/Numbers/NatInt/NZAxioms.v b/theories/Numbers/NatInt/NZAxioms.v index ee7ee159f..7cfa62eab 100644 --- a/theories/Numbers/NatInt/NZAxioms.v +++ b/theories/Numbers/NatInt/NZAxioms.v @@ -8,8 +8,6 @@ (** Initial Author : Evgeny Makarov, INRIA, 2007 *) -(*i $Id$ i*) - Require Export Equalities Orders NumPrelude GenericMinMax. (** Axiomatization of a domain with zero, successor, predecessor, diff --git a/theories/Numbers/NatInt/NZBase.v b/theories/Numbers/NatInt/NZBase.v index 18e3b9b92..9f587a1d0 100644 --- a/theories/Numbers/NatInt/NZBase.v +++ b/theories/Numbers/NatInt/NZBase.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms. Module Type NZBasePropSig (Import NZ : NZDomainSig'). diff --git a/theories/Numbers/NatInt/NZDomain.v b/theories/Numbers/NatInt/NZDomain.v index eb06cae03..7afbee4a4 100644 --- a/theories/Numbers/NatInt/NZDomain.v +++ b/theories/Numbers/NatInt/NZDomain.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export NumPrelude NZAxioms. Require Import NZBase NZOrder NZAddOrder Plus Minus. diff --git a/theories/Numbers/NatInt/NZMul.v b/theories/Numbers/NatInt/NZMul.v index 296bd095f..c97aa9f3a 100644 --- a/theories/Numbers/NatInt/NZMul.v +++ b/theories/Numbers/NatInt/NZMul.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms NZBase NZAdd. Module Type NZMulPropSig diff --git a/theories/Numbers/NatInt/NZMulOrder.v b/theories/Numbers/NatInt/NZMulOrder.v index 7b64a6983..acc43fc17 100644 --- a/theories/Numbers/NatInt/NZMulOrder.v +++ b/theories/Numbers/NatInt/NZMulOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms. Require Import NZAddOrder. diff --git a/theories/Numbers/NatInt/NZOrder.v b/theories/Numbers/NatInt/NZOrder.v index 14fa0bfde..bfbcc2c65 100644 --- a/theories/Numbers/NatInt/NZOrder.v +++ b/theories/Numbers/NatInt/NZOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NZAxioms NZBase Decidable OrdersTac. Module Type NZOrderPropSig diff --git a/theories/Numbers/NatInt/NZProperties.v b/theories/Numbers/NatInt/NZProperties.v index 125b4f62c..cc7bfe031 100644 --- a/theories/Numbers/NatInt/NZProperties.v +++ b/theories/Numbers/NatInt/NZProperties.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NZAxioms NZMulOrder. (** This functor summarizes all known facts about NZ. diff --git a/theories/Numbers/Natural/Abstract/NAdd.v b/theories/Numbers/Natural/Abstract/NAdd.v index 9f0b54a6a..859641280 100644 --- a/theories/Numbers/Natural/Abstract/NAdd.v +++ b/theories/Numbers/Natural/Abstract/NAdd.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NBase. Module NAddPropFunct (Import N : NAxiomsSig'). diff --git a/theories/Numbers/Natural/Abstract/NAddOrder.v b/theories/Numbers/Natural/Abstract/NAddOrder.v index 0ce04e54e..67bc80850 100644 --- a/theories/Numbers/Natural/Abstract/NAddOrder.v +++ b/theories/Numbers/Natural/Abstract/NAddOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NOrder. Module NAddOrderPropFunct (Import N : NAxiomsSig'). diff --git a/theories/Numbers/Natural/Abstract/NAxioms.v b/theories/Numbers/Natural/Abstract/NAxioms.v index 42016ab10..cd3d8f0a8 100644 --- a/theories/Numbers/Natural/Abstract/NAxioms.v +++ b/theories/Numbers/Natural/Abstract/NAxioms.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NZAxioms. Set Implicit Arguments. diff --git a/theories/Numbers/Natural/Abstract/NBase.v b/theories/Numbers/Natural/Abstract/NBase.v index 842f4bcf2..f26f56d0c 100644 --- a/theories/Numbers/Natural/Abstract/NBase.v +++ b/theories/Numbers/Natural/Abstract/NBase.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export Decidable. Require Export NAxioms. Require Import NZProperties. diff --git a/theories/Numbers/Natural/Abstract/NDefOps.v b/theories/Numbers/Natural/Abstract/NDefOps.v index 22eb2cb34..2302e8d35 100644 --- a/theories/Numbers/Natural/Abstract/NDefOps.v +++ b/theories/Numbers/Natural/Abstract/NDefOps.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import Bool. (* To get the orb and negb function *) Require Import RelationPairs. Require Export NStrongRec. diff --git a/theories/Numbers/Natural/Abstract/NIso.v b/theories/Numbers/Natural/Abstract/NIso.v index 47bf38cba..12dcd3258 100644 --- a/theories/Numbers/Natural/Abstract/NIso.v +++ b/theories/Numbers/Natural/Abstract/NIso.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import NBase. Module Homomorphism (N1 N2 : NAxiomsSig). diff --git a/theories/Numbers/Natural/Abstract/NMulOrder.v b/theories/Numbers/Natural/Abstract/NMulOrder.v index a2162b137..29d1838c2 100644 --- a/theories/Numbers/Natural/Abstract/NMulOrder.v +++ b/theories/Numbers/Natural/Abstract/NMulOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NAddOrder. Module NMulOrderPropFunct (Import N : NAxiomsSig'). diff --git a/theories/Numbers/Natural/Abstract/NOrder.v b/theories/Numbers/Natural/Abstract/NOrder.v index 090c02ecf..9439e04f5 100644 --- a/theories/Numbers/Natural/Abstract/NOrder.v +++ b/theories/Numbers/Natural/Abstract/NOrder.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NAdd. Module NOrderPropFunct (Import N : NAxiomsSig'). diff --git a/theories/Numbers/Natural/Abstract/NProperties.v b/theories/Numbers/Natural/Abstract/NProperties.v index 9fc9b290e..eed7cac18 100644 --- a/theories/Numbers/Natural/Abstract/NProperties.v +++ b/theories/Numbers/Natural/Abstract/NProperties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export NAxioms NMaxMin. (** This functor summarizes all known facts about N. diff --git a/theories/Numbers/Natural/Abstract/NStrongRec.v b/theories/Numbers/Natural/Abstract/NStrongRec.v index cbbcdbff5..bd666bc8b 100644 --- a/theories/Numbers/Natural/Abstract/NStrongRec.v +++ b/theories/Numbers/Natural/Abstract/NStrongRec.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - (** This file defined the strong (course-of-value, well-founded) recursion and proves its properties *) diff --git a/theories/Numbers/Natural/Abstract/NSub.v b/theories/Numbers/Natural/Abstract/NSub.v index 1df032ea3..7d3117fdb 100644 --- a/theories/Numbers/Natural/Abstract/NSub.v +++ b/theories/Numbers/Natural/Abstract/NSub.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export NMulOrder. Module Type NSubPropFunct (Import N : NAxiomsSig'). diff --git a/theories/Numbers/Natural/BigN/NMake_gen.ml b/theories/Numbers/Natural/BigN/NMake_gen.ml index 5442a5626..20cb01b16 100644 --- a/theories/Numbers/Natural/BigN/NMake_gen.ml +++ b/theories/Numbers/Natural/BigN/NMake_gen.ml @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - (*S NMake_gen.ml : this file generates NMake.v *) diff --git a/theories/Numbers/Natural/BigN/Nbasic.v b/theories/Numbers/Natural/BigN/Nbasic.v index 9772e6a1f..9177b8092 100644 --- a/theories/Numbers/Natural/BigN/Nbasic.v +++ b/theories/Numbers/Natural/BigN/Nbasic.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith. Require Import BigNumPrelude. Require Import Max. diff --git a/theories/Numbers/Natural/Binary/NBinary.v b/theories/Numbers/Natural/Binary/NBinary.v index e8651d47c..ba592507b 100644 --- a/theories/Numbers/Natural/Binary/NBinary.v +++ b/theories/Numbers/Natural/Binary/NBinary.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinPos Ndiv_def. Require Export BinNat. Require Import NAxioms NProperties NDiv. diff --git a/theories/Numbers/Natural/Peano/NPeano.v b/theories/Numbers/Natural/Peano/NPeano.v index 80d434bab..491c33666 100644 --- a/theories/Numbers/Natural/Peano/NPeano.v +++ b/theories/Numbers/Natural/Peano/NPeano.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import Peano Peano_dec Compare_dec EqNat NAxioms NProperties NDiv. (** Functions not already defined: div mod *) diff --git a/theories/Numbers/Natural/SpecViaZ/NSig.v b/theories/Numbers/Natural/SpecViaZ/NSig.v index 3f60cbf1a..55a6302aa 100644 --- a/theories/Numbers/Natural/SpecViaZ/NSig.v +++ b/theories/Numbers/Natural/SpecViaZ/NSig.v @@ -8,8 +8,6 @@ (* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith Znumtheory. Open Scope Z_scope. diff --git a/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v b/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v index 49a60916a..8cbd96c1f 100644 --- a/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v +++ b/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith Nnat NAxioms NDiv NSig. (** * The interface [NSig.NType] implies the interface [NAxiomsSig] *) diff --git a/theories/Numbers/NumPrelude.v b/theories/Numbers/NumPrelude.v index 32860cd31..5022c9ae6 100644 --- a/theories/Numbers/NumPrelude.v +++ b/theories/Numbers/NumPrelude.v @@ -8,8 +8,6 @@ (* Evgeny Makarov, INRIA, 2007 *) (************************************************************************) -(*i $Id$ i*) - Require Export Setoid Morphisms. Set Implicit Arguments. diff --git a/theories/Numbers/Rational/SpecViaQ/QSig.v b/theories/Numbers/Rational/SpecViaQ/QSig.v index 10d0189a3..6466fc511 100644 --- a/theories/Numbers/Rational/SpecViaQ/QSig.v +++ b/theories/Numbers/Rational/SpecViaQ/QSig.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import QArith Qpower Qminmax Orders RelationPairs GenericMinMax. Open Scope Q_scope. diff --git a/theories/Program/Basics.v b/theories/Program/Basics.v index 0a4b15d29..69e3206ba 100644 --- a/theories/Program/Basics.v +++ b/theories/Program/Basics.v @@ -6,8 +6,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Standard functions and combinators. Proofs about them require functional extensionality and can be found diff --git a/theories/Program/Combinators.v b/theories/Program/Combinators.v index 31661b9d3..8d041422d 100644 --- a/theories/Program/Combinators.v +++ b/theories/Program/Combinators.v @@ -6,8 +6,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** * Proofs about standard combinators, exports functional extensionality. Author: Matthieu Sozeau diff --git a/theories/Program/Equality.v b/theories/Program/Equality.v index c3c5f9c95..5a047ec5c 100644 --- a/theories/Program/Equality.v +++ b/theories/Program/Equality.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Tactics related to (dependent) equality and proof irrelevance. *) Require Export ProofIrrelevance. diff --git a/theories/Program/Program.v b/theories/Program/Program.v index cdfc78583..ffdd1bd55 100644 --- a/theories/Program/Program.v +++ b/theories/Program/Program.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Export Coq.Program.Utils. Require Export Coq.Program.Wf. Require Export Coq.Program.Equality. diff --git a/theories/Program/Subset.v b/theories/Program/Subset.v index 89f477d8f..523171013 100644 --- a/theories/Program/Subset.v +++ b/theories/Program/Subset.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Tactics related to subsets and proof irrelevance. *) Require Import Coq.Program.Utils. diff --git a/theories/Program/Syntax.v b/theories/Program/Syntax.v index 916c33ee6..2c5fb79c5 100644 --- a/theories/Program/Syntax.v +++ b/theories/Program/Syntax.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Custom notations and implicits for Coq prelude definitions. Author: Matthieu Sozeau diff --git a/theories/Program/Tactics.v b/theories/Program/Tactics.v index d187941d2..f4d53c279 100644 --- a/theories/Program/Tactics.v +++ b/theories/Program/Tactics.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This module implements various tactics used to simplify the goals produced by Program, which are also generally useful. *) diff --git a/theories/Program/Utils.v b/theories/Program/Utils.v index fbf0b03cf..dbcaea80f 100644 --- a/theories/Program/Utils.v +++ b/theories/Program/Utils.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Various syntaxic shortands that are useful with [Program]. *) Require Export Coq.Program.Tactics. diff --git a/theories/Program/Wf.v b/theories/Program/Wf.v index c4d06fd72..70a6fe97a 100644 --- a/theories/Program/Wf.v +++ b/theories/Program/Wf.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Reformulation of the Wf module using subsets where possible, providing the support for [Program]'s treatment of well-founded definitions. *) diff --git a/theories/QArith/QArith.v b/theories/QArith/QArith.v index f7a28598e..fe1ff3674 100644 --- a/theories/QArith/QArith.v +++ b/theories/QArith/QArith.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export QArith_base. Require Export Qring. Require Export Qreduction. diff --git a/theories/QArith/QArith_base.v b/theories/QArith/QArith_base.v index 609241d5e..111d2391a 100644 --- a/theories/QArith/QArith_base.v +++ b/theories/QArith/QArith_base.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export ZArith. Require Export ZArithRing. Require Export Morphisms Setoid Bool. diff --git a/theories/QArith/Qcanon.v b/theories/QArith/Qcanon.v index 34d6267e3..b26b828ca 100644 --- a/theories/QArith/Qcanon.v +++ b/theories/QArith/Qcanon.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Field. Require Import QArith. Require Import Znumtheory. diff --git a/theories/QArith/Qfield.v b/theories/QArith/Qfield.v index fbfae55c3..524996c38 100644 --- a/theories/QArith/Qfield.v +++ b/theories/QArith/Qfield.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Field. Require Export QArith_base. Require Import NArithRing. diff --git a/theories/QArith/Qreals.v b/theories/QArith/Qreals.v index 12e371ee9..15fea8516 100644 --- a/theories/QArith/Qreals.v +++ b/theories/QArith/Qreals.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Rbase. Require Export QArith_base. diff --git a/theories/QArith/Qreduction.v b/theories/QArith/Qreduction.v index 27e3c4e02..4f16f5b8c 100644 --- a/theories/QArith/Qreduction.v +++ b/theories/QArith/Qreduction.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Normalisation functions for rational numbers. *) Require Export QArith_base. diff --git a/theories/QArith/Qring.v b/theories/QArith/Qring.v index 8c9e2dfa3..96ed046a6 100644 --- a/theories/QArith/Qring.v +++ b/theories/QArith/Qring.v @@ -6,6 +6,4 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Qfield. diff --git a/theories/Reals/Alembert.v b/theories/Reals/Alembert.v index ef75323e0..1b9be0795 100644 --- a/theories/Reals/Alembert.v +++ b/theories/Reals/Alembert.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/AltSeries.v b/theories/Reals/AltSeries.v index cccc8ceec..9c29e26a3 100644 --- a/theories/Reals/AltSeries.v +++ b/theories/Reals/AltSeries.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) - (*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/ArithProp.v b/theories/Reals/ArithProp.v index f22ff5cb2..48324e8e8 100644 --- a/theories/Reals/ArithProp.v +++ b/theories/Reals/ArithProp.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) - (*i $Id$ i*) - Require Import Rbase. Require Import Rbasic_fun. Require Import Even. diff --git a/theories/Reals/Binomial.v b/theories/Reals/Binomial.v index 0d34d22c5..d0df984a1 100644 --- a/theories/Reals/Binomial.v +++ b/theories/Reals/Binomial.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) - (*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import PartSum. diff --git a/theories/Reals/Cauchy_prod.v b/theories/Reals/Cauchy_prod.v index 6ea0767d0..68a842c9f 100644 --- a/theories/Reals/Cauchy_prod.v +++ b/theories/Reals/Cauchy_prod.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) - (*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/Cos_plus.v b/theories/Reals/Cos_plus.v index 6c08356a7..c5e2c0ed3 100644 --- a/theories/Reals/Cos_plus.v +++ b/theories/Reals/Cos_plus.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) - (*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Cos_rel.v b/theories/Reals/Cos_rel.v index 7a893c53c..d27e0ae4c 100644 --- a/theories/Reals/Cos_rel.v +++ b/theories/Reals/Cos_rel.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/DiscrR.v b/theories/Reals/DiscrR.v index e037c77b5..0d41b5900 100644 --- a/theories/Reals/DiscrR.v +++ b/theories/Reals/DiscrR.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import RIneq. Require Import Omega. Open Local Scope R_scope. diff --git a/theories/Reals/Exp_prop.v b/theories/Reals/Exp_prop.v index 1c74f55a0..287057f0f 100644 --- a/theories/Reals/Exp_prop.v +++ b/theories/Reals/Exp_prop.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Integration.v b/theories/Reals/Integration.v index 774a0bd5c..eba81ff9b 100644 --- a/theories/Reals/Integration.v +++ b/theories/Reals/Integration.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export NewtonInt. Require Export RiemannInt_SF. Require Export RiemannInt. \ No newline at end of file diff --git a/theories/Reals/LegacyRfield.v b/theories/Reals/LegacyRfield.v index b33274af9..ca7cb8fea 100644 --- a/theories/Reals/LegacyRfield.v +++ b/theories/Reals/LegacyRfield.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Raxioms. Require Export LegacyField. Import LegacyRing_theory. diff --git a/theories/Reals/MVT.v b/theories/Reals/MVT.v index 4037e3dec..72bd62a69 100644 --- a/theories/Reals/MVT.v +++ b/theories/Reals/MVT.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis1. diff --git a/theories/Reals/NewtonInt.v b/theories/Reals/NewtonInt.v index 74bcf7dcd..0d75a9dee 100644 --- a/theories/Reals/NewtonInt.v +++ b/theories/Reals/NewtonInt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/PSeries_reg.v b/theories/Reals/PSeries_reg.v index 97793386d..80a5b87a8 100644 --- a/theories/Reals/PSeries_reg.v +++ b/theories/Reals/PSeries_reg.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/PartSum.v b/theories/Reals/PartSum.v index 6a33b8092..e9a224b97 100644 --- a/theories/Reals/PartSum.v +++ b/theories/Reals/PartSum.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/RIneq.v b/theories/Reals/RIneq.v index 2b6af10ec..7c4555605 100644 --- a/theories/Reals/RIneq.v +++ b/theories/Reals/RIneq.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** * Basic lemmas for the classical real numbers *) (*********************************************************) diff --git a/theories/Reals/RList.v b/theories/Reals/RList.v index 545bd68b2..8cf56cd7b 100644 --- a/theories/Reals/RList.v +++ b/theories/Reals/RList.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Open Local Scope R_scope. diff --git a/theories/Reals/R_Ifp.v b/theories/Reals/R_Ifp.v index 57b2c7675..e530070b1 100644 --- a/theories/Reals/R_Ifp.v +++ b/theories/Reals/R_Ifp.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (**********************************************************) (** Complements for the reals.Integer and fractional part *) (* *) diff --git a/theories/Reals/R_sqr.v b/theories/Reals/R_sqr.v index 6460a9271..1cccb8848 100644 --- a/theories/Reals/R_sqr.v +++ b/theories/Reals/R_sqr.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rbasic_fun. Open Local Scope R_scope. diff --git a/theories/Reals/R_sqrt.v b/theories/Reals/R_sqrt.v index 2c43ee9b9..13232566f 100644 --- a/theories/Reals/R_sqrt.v +++ b/theories/Reals/R_sqrt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rsqrt_def. diff --git a/theories/Reals/Ranalysis.v b/theories/Reals/Ranalysis.v index 500dd5295..53267174b 100644 --- a/theories/Reals/Ranalysis.v +++ b/theories/Reals/Ranalysis.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rtrigo. diff --git a/theories/Reals/Ranalysis1.v b/theories/Reals/Ranalysis1.v index 1516b3384..a0b10c891 100644 --- a/theories/Reals/Ranalysis1.v +++ b/theories/Reals/Ranalysis1.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Export Rlimit. diff --git a/theories/Reals/Ranalysis2.v b/theories/Reals/Ranalysis2.v index 1d44b3e73..04c00cb30 100644 --- a/theories/Reals/Ranalysis2.v +++ b/theories/Reals/Ranalysis2.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis1. diff --git a/theories/Reals/Ranalysis3.v b/theories/Reals/Ranalysis3.v index 3b685cd8a..28da1c7c4 100644 --- a/theories/Reals/Ranalysis3.v +++ b/theories/Reals/Ranalysis3.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis1. diff --git a/theories/Reals/Ranalysis4.v b/theories/Reals/Ranalysis4.v index 1ed3fb713..abf0b883f 100644 --- a/theories/Reals/Ranalysis4.v +++ b/theories/Reals/Ranalysis4.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Raxioms.v b/theories/Reals/Raxioms.v index 9715414f5..1ed75cdb6 100644 --- a/theories/Reals/Raxioms.v +++ b/theories/Reals/Raxioms.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** Axiomatisation of the classical reals *) (*********************************************************) diff --git a/theories/Reals/Rbase.v b/theories/Reals/Rbase.v index ab1c07474..8843c5e6e 100644 --- a/theories/Reals/Rbase.v +++ b/theories/Reals/Rbase.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Rdefinitions. Require Export Raxioms. Require Export RIneq. diff --git a/theories/Reals/Rbasic_fun.v b/theories/Reals/Rbasic_fun.v index 7588020c5..2e1bd0797 100644 --- a/theories/Reals/Rbasic_fun.v +++ b/theories/Reals/Rbasic_fun.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** Complements for the real numbers *) (* *) diff --git a/theories/Reals/Rcomplete.v b/theories/Reals/Rcomplete.v index 27d5c49ef..de3250529 100644 --- a/theories/Reals/Rcomplete.v +++ b/theories/Reals/Rcomplete.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/Rdefinitions.v b/theories/Reals/Rdefinitions.v index 023cfc93c..ab6ed8b10 100644 --- a/theories/Reals/Rdefinitions.v +++ b/theories/Reals/Rdefinitions.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** Definitions for the axiomatization *) diff --git a/theories/Reals/Rderiv.v b/theories/Reals/Rderiv.v index 6413943a9..19ebcd3cb 100644 --- a/theories/Reals/Rderiv.v +++ b/theories/Reals/Rderiv.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** Definition of the derivative,continuity *) (* *) diff --git a/theories/Reals/Reals.v b/theories/Reals/Reals.v index d18213db4..de57a5af2 100644 --- a/theories/Reals/Reals.v +++ b/theories/Reals/Reals.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** The library REALS is divided in 6 parts : - Rbase: basic lemmas on R equalities and inequalities diff --git a/theories/Reals/Rfunctions.v b/theories/Reals/Rfunctions.v index 7371c8acf..668891369 100644 --- a/theories/Reals/Rfunctions.v +++ b/theories/Reals/Rfunctions.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i Some properties about pow and sum have been made with John Harrison i*) (*i Some Lemmas (about pow and powerRZ) have been done by Laurent Thery i*) diff --git a/theories/Reals/Rgeom.v b/theories/Reals/Rgeom.v index 8890cbb50..dceb98d45 100644 --- a/theories/Reals/Rgeom.v +++ b/theories/Reals/Rgeom.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/RiemannInt.v b/theories/Reals/RiemannInt.v index 9fd6e0088..abf817d7a 100644 --- a/theories/Reals/RiemannInt.v +++ b/theories/Reals/RiemannInt.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rfunctions. Require Import SeqSeries. Require Import Ranalysis. diff --git a/theories/Reals/RiemannInt_SF.v b/theories/Reals/RiemannInt_SF.v index f9b1b890f..f783d1d82 100644 --- a/theories/Reals/RiemannInt_SF.v +++ b/theories/Reals/RiemannInt_SF.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis. diff --git a/theories/Reals/Rlimit.v b/theories/Reals/Rlimit.v index 3aaa7300a..e0f47364f 100644 --- a/theories/Reals/Rlimit.v +++ b/theories/Reals/Rlimit.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************) (** Definition of the limit *) (* *) diff --git a/theories/Reals/Rpow_def.v b/theories/Reals/Rpow_def.v index c7d1893be..f922e25f6 100644 --- a/theories/Reals/Rpow_def.v +++ b/theories/Reals/Rpow_def.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import Rdefinitions. Fixpoint pow (r:R) (n:nat) : R := diff --git a/theories/Reals/Rpower.v b/theories/Reals/Rpower.v index a4feed8f3..957466cbe 100644 --- a/theories/Reals/Rpower.v +++ b/theories/Reals/Rpower.v @@ -6,7 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) (*i Due to L.Thery i*) (************************************************************) diff --git a/theories/Reals/Rprod.v b/theories/Reals/Rprod.v index bb3df6bb8..4e3f4d089 100644 --- a/theories/Reals/Rprod.v +++ b/theories/Reals/Rprod.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Compare. Require Import Rbase. Require Import Rfunctions. diff --git a/theories/Reals/Rseries.v b/theories/Reals/Rseries.v index 1ed6b03c5..9e5122062 100644 --- a/theories/Reals/Rseries.v +++ b/theories/Reals/Rseries.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Compare. diff --git a/theories/Reals/Rsigma.v b/theories/Reals/Rsigma.v index 917592702..155577746 100644 --- a/theories/Reals/Rsigma.v +++ b/theories/Reals/Rsigma.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/Rsqrt_def.v b/theories/Reals/Rsqrt_def.v index 33c20355c..a8f12a6b3 100644 --- a/theories/Reals/Rsqrt_def.v +++ b/theories/Reals/Rsqrt_def.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Sumbool. Require Import Rbase. Require Import Rfunctions. diff --git a/theories/Reals/Rtopology.v b/theories/Reals/Rtopology.v index 5b55896b1..a086cfd46 100644 --- a/theories/Reals/Rtopology.v +++ b/theories/Reals/Rtopology.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis1. diff --git a/theories/Reals/Rtrigo.v b/theories/Reals/Rtrigo.v index 4981d6fdf..582b6be75 100644 --- a/theories/Reals/Rtrigo.v +++ b/theories/Reals/Rtrigo.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Rtrigo_alt.v b/theories/Reals/Rtrigo_alt.v index fe2da8391..1cf0944c0 100644 --- a/theories/Reals/Rtrigo_alt.v +++ b/theories/Reals/Rtrigo_alt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Rtrigo_calc.v b/theories/Reals/Rtrigo_calc.v index a7fddb473..33ea1adba 100644 --- a/theories/Reals/Rtrigo_calc.v +++ b/theories/Reals/Rtrigo_calc.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Rtrigo_def.v b/theories/Reals/Rtrigo_def.v index 9588e4438..265dae9d4 100644 --- a/theories/Reals/Rtrigo_def.v +++ b/theories/Reals/Rtrigo_def.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Rtrigo_fun.v b/theories/Reals/Rtrigo_fun.v index cb53b5346..62d8d9f5f 100644 --- a/theories/Reals/Rtrigo_fun.v +++ b/theories/Reals/Rtrigo_fun.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/Rtrigo_reg.v b/theories/Reals/Rtrigo_reg.v index 5b731488b..f38e59e82 100644 --- a/theories/Reals/Rtrigo_reg.v +++ b/theories/Reals/Rtrigo_reg.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import SeqSeries. diff --git a/theories/Reals/SeqProp.v b/theories/Reals/SeqProp.v index 82647c837..642e7fc9e 100644 --- a/theories/Reals/SeqProp.v +++ b/theories/Reals/SeqProp.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Rseries. diff --git a/theories/Reals/SeqSeries.v b/theories/Reals/SeqSeries.v index dbfc85bb9..dcfadd566 100644 --- a/theories/Reals/SeqSeries.v +++ b/theories/Reals/SeqSeries.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Max. diff --git a/theories/Reals/SplitAbsolu.v b/theories/Reals/SplitAbsolu.v index 5882f953c..90048e50d 100644 --- a/theories/Reals/SplitAbsolu.v +++ b/theories/Reals/SplitAbsolu.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbasic_fun. Ltac split_case_Rabs := diff --git a/theories/Reals/SplitRmult.v b/theories/Reals/SplitRmult.v index 51e54860d..322808f9b 100644 --- a/theories/Reals/SplitRmult.v +++ b/theories/Reals/SplitRmult.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i Lemma mult_non_zero :(r1,r2:R)``r1<>0`` /\ ``r2<>0`` -> ``r1*r2<>0``. i*) diff --git a/theories/Reals/Sqrt_reg.v b/theories/Reals/Sqrt_reg.v index 4f336648b..3961b8b0c 100644 --- a/theories/Reals/Sqrt_reg.v +++ b/theories/Reals/Sqrt_reg.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Rbase. Require Import Rfunctions. Require Import Ranalysis1. diff --git a/theories/Relations/Operators_Properties.v b/theories/Relations/Operators_Properties.v index 1976b435c..cfb952632 100644 --- a/theories/Relations/Operators_Properties.v +++ b/theories/Relations/Operators_Properties.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (************************************************************************) (** * Some properties of the operators on relations *) (************************************************************************) diff --git a/theories/Relations/Relation_Definitions.v b/theories/Relations/Relation_Definitions.v index c03c4b95f..4f676484a 100644 --- a/theories/Relations/Relation_Definitions.v +++ b/theories/Relations/Relation_Definitions.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Section Relation_Definition. Variable A : Type. diff --git a/theories/Relations/Relation_Operators.v b/theories/Relations/Relation_Operators.v index 39e0331d5..bdc44dd17 100644 --- a/theories/Relations/Relation_Operators.v +++ b/theories/Relations/Relation_Operators.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (************************************************************************) (** * Bruno Barras, Cristina Cornes *) (** * *) diff --git a/theories/Relations/Relations.v b/theories/Relations/Relations.v index 1c6df08a4..f1e20b10e 100644 --- a/theories/Relations/Relations.v +++ b/theories/Relations/Relations.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Relation_Definitions. Require Export Relation_Operators. Require Export Operators_Properties. diff --git a/theories/Setoids/Setoid.v b/theories/Setoids/Setoid.v index c5530e7ca..cf641253a 100644 --- a/theories/Setoids/Setoid.v +++ b/theories/Setoids/Setoid.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$: i*) - Require Export Coq.Classes.SetoidTactics. Export Morphisms.ProperNotations. diff --git a/theories/Sets/Classical_sets.v b/theories/Sets/Classical_sets.v index 5f6860997..5fbfadd4c 100644 --- a/theories/Sets/Classical_sets.v +++ b/theories/Sets/Classical_sets.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Constructive_sets. Require Export Classical_Type. diff --git a/theories/Sets/Constructive_sets.v b/theories/Sets/Constructive_sets.v index 0719365f1..294dbb0cd 100644 --- a/theories/Sets/Constructive_sets.v +++ b/theories/Sets/Constructive_sets.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Section Ensembles_facts. diff --git a/theories/Sets/Cpo.v b/theories/Sets/Cpo.v index 8c69e6877..6d537f59b 100644 --- a/theories/Sets/Cpo.v +++ b/theories/Sets/Cpo.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Relations_1. Require Export Partial_Order. diff --git a/theories/Sets/Ensembles.v b/theories/Sets/Ensembles.v index 0fa9c74a8..8843cadd6 100644 --- a/theories/Sets/Ensembles.v +++ b/theories/Sets/Ensembles.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Section Ensembles. Variable U : Type. diff --git a/theories/Sets/Finite_sets.v b/theories/Sets/Finite_sets.v index 019c25a55..11ac3b9e4 100644 --- a/theories/Sets/Finite_sets.v +++ b/theories/Sets/Finite_sets.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Import Ensembles. Section Ensembles_finis. diff --git a/theories/Sets/Finite_sets_facts.v b/theories/Sets/Finite_sets_facts.v index fdcc4150f..da4a35813 100644 --- a/theories/Sets/Finite_sets_facts.v +++ b/theories/Sets/Finite_sets_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Finite_sets. Require Export Constructive_sets. Require Export Classical_Type. diff --git a/theories/Sets/Image.v b/theories/Sets/Image.v index 64c341bd3..313a18dcc 100644 --- a/theories/Sets/Image.v +++ b/theories/Sets/Image.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Finite_sets. Require Export Constructive_sets. Require Export Classical_Type. diff --git a/theories/Sets/Infinite_sets.v b/theories/Sets/Infinite_sets.v index b63ec1d47..0ae11b4f6 100644 --- a/theories/Sets/Infinite_sets.v +++ b/theories/Sets/Infinite_sets.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Finite_sets. Require Export Constructive_sets. Require Export Classical_Type. diff --git a/theories/Sets/Integers.v b/theories/Sets/Integers.v index 15c1b665e..8fe9928b1 100644 --- a/theories/Sets/Integers.v +++ b/theories/Sets/Integers.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Finite_sets. Require Export Constructive_sets. Require Export Classical_Type. diff --git a/theories/Sets/Multiset.v b/theories/Sets/Multiset.v index 7216ae335..5b7aa24b7 100644 --- a/theories/Sets/Multiset.v +++ b/theories/Sets/Multiset.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* G. Huet 1-9-95 *) Require Import Permut Setoid. diff --git a/theories/Sets/Partial_Order.v b/theories/Sets/Partial_Order.v index 4fe8f4f6a..195f454e5 100644 --- a/theories/Sets/Partial_Order.v +++ b/theories/Sets/Partial_Order.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Relations_1. diff --git a/theories/Sets/Permut.v b/theories/Sets/Permut.v index f593031a0..25a121cb3 100644 --- a/theories/Sets/Permut.v +++ b/theories/Sets/Permut.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* G. Huet 1-9-95 *) (** We consider a Set [U], given with a commutative-associative operator [op], diff --git a/theories/Sets/Powerset.v b/theories/Sets/Powerset.v index c323ca356..9ecb600a5 100644 --- a/theories/Sets/Powerset.v +++ b/theories/Sets/Powerset.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Relations_1. Require Export Relations_1_facts. diff --git a/theories/Sets/Powerset_Classical_facts.v b/theories/Sets/Powerset_Classical_facts.v index 36d2150c3..8f881c363 100644 --- a/theories/Sets/Powerset_Classical_facts.v +++ b/theories/Sets/Powerset_Classical_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Constructive_sets. Require Export Relations_1. diff --git a/theories/Sets/Powerset_facts.v b/theories/Sets/Powerset_facts.v index 76f7f1ec8..61f783957 100644 --- a/theories/Sets/Powerset_facts.v +++ b/theories/Sets/Powerset_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Ensembles. Require Export Constructive_sets. Require Export Relations_1. diff --git a/theories/Sets/Relations_1.v b/theories/Sets/Relations_1.v index 85d0cffcc..eb3273959 100644 --- a/theories/Sets/Relations_1.v +++ b/theories/Sets/Relations_1.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Section Relations_1. Variable U : Type. diff --git a/theories/Sets/Relations_1_facts.v b/theories/Sets/Relations_1_facts.v index fd83b0e0d..484245bc8 100644 --- a/theories/Sets/Relations_1_facts.v +++ b/theories/Sets/Relations_1_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Relations_1. Definition Complement (U:Type) (R:Relation U) : Relation U := diff --git a/theories/Sets/Relations_2.v b/theories/Sets/Relations_2.v index 11ac85e84..3b1e7057d 100644 --- a/theories/Sets/Relations_2.v +++ b/theories/Sets/Relations_2.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Relations_1. Section Relations_2. diff --git a/theories/Sets/Relations_2_facts.v b/theories/Sets/Relations_2_facts.v index 3554901b9..6fd07160f 100644 --- a/theories/Sets/Relations_2_facts.v +++ b/theories/Sets/Relations_2_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Relations_1. Require Export Relations_1_facts. Require Export Relations_2. diff --git a/theories/Sets/Relations_3.v b/theories/Sets/Relations_3.v index 970db1827..991b38242 100644 --- a/theories/Sets/Relations_3.v +++ b/theories/Sets/Relations_3.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Relations_1. Require Export Relations_2. diff --git a/theories/Sets/Relations_3_facts.v b/theories/Sets/Relations_3_facts.v index d8bf7dc3c..a2a0f4584 100644 --- a/theories/Sets/Relations_3_facts.v +++ b/theories/Sets/Relations_3_facts.v @@ -24,8 +24,6 @@ (* in Summer 1995. Several developments by E. Ledinot were an inspiration. *) (****************************************************************************) -(*i $Id$ i*) - Require Export Relations_1. Require Export Relations_1_facts. Require Export Relations_2. diff --git a/theories/Sets/Uniset.v b/theories/Sets/Uniset.v index 909c79838..41e7f0edf 100644 --- a/theories/Sets/Uniset.v +++ b/theories/Sets/Uniset.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Sets as characteristic functions *) (* G. Huet 1-9-95 *) diff --git a/theories/Sorting/Heap.v b/theories/Sorting/Heap.v index 4124ef983..c48d22d62 100644 --- a/theories/Sorting/Heap.v +++ b/theories/Sorting/Heap.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file is deprecated, for a tree on list, use [Mergesort.v]. *) (** A development of Treesort on Heap trees. It has an average diff --git a/theories/Sorting/Mergesort.v b/theories/Sorting/Mergesort.v index 238013b85..5830fabe4 100644 --- a/theories/Sorting/Mergesort.v +++ b/theories/Sorting/Mergesort.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** A modular implementation of mergesort (the complexity is O(n.log n) in the length of the list) *) diff --git a/theories/Sorting/PermutEq.v b/theories/Sorting/PermutEq.v index 8e6aa6dce..6ad0b6ba0 100644 --- a/theories/Sorting/PermutEq.v +++ b/theories/Sorting/PermutEq.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Relations Setoid SetoidList List Multiset PermutSetoid Permutation. Set Implicit Arguments. diff --git a/theories/Sorting/PermutSetoid.v b/theories/Sorting/PermutSetoid.v index 203e212b6..5faaebe28 100644 --- a/theories/Sorting/PermutSetoid.v +++ b/theories/Sorting/PermutSetoid.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Omega Relations Multiset SetoidList. (** This file is deprecated, use [Permutation.v] instead. diff --git a/theories/Sorting/Permutation.v b/theories/Sorting/Permutation.v index c3cd4f4a8..e861b9ce7 100644 --- a/theories/Sorting/Permutation.v +++ b/theories/Sorting/Permutation.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*********************************************************************) (** ** List permutations as a composition of adjacent transpositions *) (*********************************************************************) diff --git a/theories/Sorting/Sorted.v b/theories/Sorting/Sorted.v index d87259eec..931e29bf8 100644 --- a/theories/Sorting/Sorted.v +++ b/theories/Sorting/Sorted.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Made by Hugo Herbelin *) (** This file defines two notions of sorted list: diff --git a/theories/Sorting/Sorting.v b/theories/Sorting/Sorting.v index 5f8da6a4d..f05cc473b 100644 --- a/theories/Sorting/Sorting.v +++ b/theories/Sorting/Sorting.v @@ -6,7 +6,5 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Sorted. Require Export Mergesort. diff --git a/theories/Strings/Ascii.v b/theories/Strings/Ascii.v index 1f90c06cf..ba01f3d4c 100644 --- a/theories/Strings/Ascii.v +++ b/theories/Strings/Ascii.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Contributed by Laurent Théry (INRIA); Adapted to Coq V8 by the Coq Development Team *) diff --git a/theories/Strings/String.v b/theories/Strings/String.v index 15f298218..c6bf9e119 100644 --- a/theories/Strings/String.v +++ b/theories/Strings/String.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Contributed by Laurent Théry (INRIA); Adapted to Coq V8 by the Coq Development Team *) diff --git a/theories/Structures/DecidableType.v b/theories/Structures/DecidableType.v index 2c72e30b1..79e817717 100644 --- a/theories/Structures/DecidableType.v +++ b/theories/Structures/DecidableType.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export SetoidList. Require Equalities. diff --git a/theories/Structures/DecidableTypeEx.v b/theories/Structures/DecidableTypeEx.v index 4407ead41..2c02f8ddd 100644 --- a/theories/Structures/DecidableTypeEx.v +++ b/theories/Structures/DecidableTypeEx.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Import DecidableType OrderedType OrderedTypeEx. Set Implicit Arguments. Unset Strict Implicit. diff --git a/theories/Structures/Equalities.v b/theories/Structures/Equalities.v index 3d4430b9e..0a6dba982 100644 --- a/theories/Structures/Equalities.v +++ b/theories/Structures/Equalities.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export RelationClasses. Set Implicit Arguments. diff --git a/theories/Structures/OrderedType.v b/theories/Structures/OrderedType.v index 72fbe7968..6b9007fdd 100644 --- a/theories/Structures/OrderedType.v +++ b/theories/Structures/OrderedType.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export SetoidList Morphisms OrdersTac. Set Implicit Arguments. Unset Strict Implicit. diff --git a/theories/Structures/OrderedTypeAlt.v b/theories/Structures/OrderedTypeAlt.v index 23ae4c85a..b054496e9 100644 --- a/theories/Structures/OrderedTypeAlt.v +++ b/theories/Structures/OrderedTypeAlt.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Import OrderedType. (** * An alternative (but equivalent) presentation for an Ordered Type diff --git a/theories/Structures/OrderedTypeEx.v b/theories/Structures/OrderedTypeEx.v index a39f336a5..600eabf11 100644 --- a/theories/Structures/OrderedTypeEx.v +++ b/theories/Structures/OrderedTypeEx.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Import OrderedType. Require Import ZArith. Require Import Omega. diff --git a/theories/Structures/Orders.v b/theories/Structures/Orders.v index 96daca5cd..d7bdfbf71 100644 --- a/theories/Structures/Orders.v +++ b/theories/Structures/Orders.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - Require Export Relations Morphisms Setoid Equalities. Set Implicit Arguments. Unset Strict Implicit. diff --git a/theories/Structures/OrdersAlt.v b/theories/Structures/OrdersAlt.v index d86b02a15..85e7fb176 100644 --- a/theories/Structures/OrdersAlt.v +++ b/theories/Structures/OrdersAlt.v @@ -11,8 +11,6 @@ * Institution: LRI, CNRS UMR 8623 - Université Paris Sud * 91405 Orsay, France *) -(* $Id$ *) - Require Import OrderedType Orders. Set Implicit Arguments. diff --git a/theories/Structures/OrdersEx.v b/theories/Structures/OrdersEx.v index b0702f681..f8a08bf4e 100644 --- a/theories/Structures/OrdersEx.v +++ b/theories/Structures/OrdersEx.v @@ -11,8 +11,6 @@ * Institution: LRI, CNRS UMR 8623 - Université Paris Sud * 91405 Orsay, France *) -(* $Id$ *) - Require Import Orders NPeano POrderedType NArith ZArith RelationPairs EqualitiesFacts. diff --git a/theories/Wellfounded/Disjoint_Union.v b/theories/Wellfounded/Disjoint_Union.v index 785d623b4..f856c8624 100644 --- a/theories/Wellfounded/Disjoint_Union.v +++ b/theories/Wellfounded/Disjoint_Union.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Cristina Cornes From : Constructing Recursion Operators in Type Theory L. Paulson JSC (1986) 2, 325-355 *) diff --git a/theories/Wellfounded/Inclusion.v b/theories/Wellfounded/Inclusion.v index 01049989e..4d7139a51 100644 --- a/theories/Wellfounded/Inclusion.v +++ b/theories/Wellfounded/Inclusion.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Bruno Barras *) Require Import Relation_Definitions. diff --git a/theories/Wellfounded/Inverse_Image.v b/theories/Wellfounded/Inverse_Image.v index c57e70725..6f7a310d5 100644 --- a/theories/Wellfounded/Inverse_Image.v +++ b/theories/Wellfounded/Inverse_Image.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Bruno Barras *) Section Inverse_Image. diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v index ff1889000..378b47184 100644 --- a/theories/Wellfounded/Lexicographic_Exponentiation.v +++ b/theories/Wellfounded/Lexicographic_Exponentiation.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Cristina Cornes From : Constructing Recursion Operators in Type Theory diff --git a/theories/Wellfounded/Lexicographic_Product.v b/theories/Wellfounded/Lexicographic_Product.v index 5144c0bee..e52c3acae 100644 --- a/theories/Wellfounded/Lexicographic_Product.v +++ b/theories/Wellfounded/Lexicographic_Product.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Authors: Bruno Barras, Cristina Cornes *) Require Import Eqdep. diff --git a/theories/Wellfounded/Transitive_Closure.v b/theories/Wellfounded/Transitive_Closure.v index c999b58ee..a6092fe37 100644 --- a/theories/Wellfounded/Transitive_Closure.v +++ b/theories/Wellfounded/Transitive_Closure.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Bruno Barras *) Require Import Relation_Definitions. diff --git a/theories/Wellfounded/Union.v b/theories/Wellfounded/Union.v index fbb3d9e3c..dbc36e3b1 100644 --- a/theories/Wellfounded/Union.v +++ b/theories/Wellfounded/Union.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Bruno Barras *) Require Import Relation_Operators. diff --git a/theories/Wellfounded/Well_Ordering.v b/theories/Wellfounded/Well_Ordering.v index e11b89248..8a5bf57f0 100644 --- a/theories/Wellfounded/Well_Ordering.v +++ b/theories/Wellfounded/Well_Ordering.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Author: Cristina Cornes. From: Constructing Recursion Operators in Type Theory L. Paulson JSC (1986) 2, 325-355 *) diff --git a/theories/Wellfounded/Wellfounded.v b/theories/Wellfounded/Wellfounded.v index fe05d61ed..77c676fc6 100644 --- a/theories/Wellfounded/Wellfounded.v +++ b/theories/Wellfounded/Wellfounded.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Export Disjoint_Union. Require Export Inclusion. Require Export Inverse_Image. diff --git a/theories/ZArith/BinInt.v b/theories/ZArith/BinInt.v index 2807532ca..06adc620f 100644 --- a/theories/ZArith/BinInt.v +++ b/theories/ZArith/BinInt.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (***********************************************************) (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) (***********************************************************) diff --git a/theories/ZArith/Int.v b/theories/ZArith/Int.v index 30c08fdc1..3a0d7090d 100644 --- a/theories/ZArith/Int.v +++ b/theories/ZArith/Int.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id$ *) - (** * An light axiomatization of integers (used in FSetAVL). *) (** We define a signature for an integer datatype based on [Z]. diff --git a/theories/ZArith/Wf_Z.v b/theories/ZArith/Wf_Z.v index 46f64c88d..7bbab9aaf 100644 --- a/theories/ZArith/Wf_Z.v +++ b/theories/ZArith/Wf_Z.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinInt. Require Import Zcompare. Require Import Zorder. diff --git a/theories/ZArith/ZArith.v b/theories/ZArith/ZArith.v index 7a68bd511..dba123091 100644 --- a/theories/ZArith/ZArith.v +++ b/theories/ZArith/ZArith.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Library for manipulating integers based on binary encoding *) Require Export ZArith_base. diff --git a/theories/ZArith/ZArith_base.v b/theories/ZArith/ZArith_base.v index cd866c375..ac86f50f6 100644 --- a/theories/ZArith/ZArith_base.v +++ b/theories/ZArith/ZArith_base.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (** Library for manipulating integers based on binary encoding. These are the basic modules, required by [Omega] and [Ring] for instance. The full library is [ZArith]. *) diff --git a/theories/ZArith/ZArith_dec.v b/theories/ZArith/ZArith_dec.v index 6e69350db..2dce5fbe4 100644 --- a/theories/ZArith/ZArith_dec.v +++ b/theories/ZArith/ZArith_dec.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Sumbool. Require Import BinInt. diff --git a/theories/ZArith/Zabs.v b/theories/ZArith/Zabs.v index ba454c327..517973a1e 100644 --- a/theories/ZArith/Zabs.v +++ b/theories/ZArith/Zabs.v @@ -6,8 +6,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Binary Integers (Pierre Crégut (CNET, Lannion, France) *) Require Import Arith_base. diff --git a/theories/ZArith/Zbool.v b/theories/ZArith/Zbool.v index 8cdd73cc7..61d706b23 100644 --- a/theories/ZArith/Zbool.v +++ b/theories/ZArith/Zbool.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import BinInt. Require Import Zeven. Require Import Zorder. diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v index 08cc564de..103c2c9d5 100644 --- a/theories/ZArith/Zcomplements.v +++ b/theories/ZArith/Zcomplements.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArithRing. Require Import ZArith_base. Require Export Omega. diff --git a/theories/ZArith/Zdigits.v b/theories/ZArith/Zdigits.v index 0a6c94986..f30d46cf3 100644 --- a/theories/ZArith/Zdigits.v +++ b/theories/ZArith/Zdigits.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Bit vectors interpreted as integers. Contribution by Jean Duprat (ENS Lyon). *) diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v index 66e275b61..0cd5bed86 100644 --- a/theories/ZArith/Zdiv.v +++ b/theories/ZArith/Zdiv.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Contribution by Claude Marché and Xavier Urbain *) (** Euclidean Division diff --git a/theories/ZArith/Zeven.v b/theories/ZArith/Zeven.v index 091310439..4dfce35ce 100644 --- a/theories/ZArith/Zeven.v +++ b/theories/ZArith/Zeven.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import BinInt. Open Scope Z_scope. diff --git a/theories/ZArith/Zgcd_alt.v b/theories/ZArith/Zgcd_alt.v index 447f6101a..f65a8f53b 100644 --- a/theories/ZArith/Zgcd_alt.v +++ b/theories/ZArith/Zgcd_alt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** * Zgcd_alt : an alternate version of Zgcd, based on Euler's algorithm *) (** diff --git a/theories/ZArith/Zhints.v b/theories/ZArith/Zhints.v index 5459e693d..d3d3eff0d 100644 --- a/theories/ZArith/Zhints.v +++ b/theories/ZArith/Zhints.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** This file centralizes the lemmas about [Z], classifying them according to the way they can be used in automatic search *) diff --git a/theories/ZArith/Zlogarithm.v b/theories/ZArith/Zlogarithm.v index 70a959c2a..397a8ab93 100644 --- a/theories/ZArith/Zlogarithm.v +++ b/theories/ZArith/Zlogarithm.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (**********************************************************************) (** The integer logarithms with base 2. diff --git a/theories/ZArith/Zmax.v b/theories/ZArith/Zmax.v index 1d9b1f108..b9ff036aa 100644 --- a/theories/ZArith/Zmax.v +++ b/theories/ZArith/Zmax.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** THIS FILE IS DEPRECATED. Use [ZBinary.Z] instead. *) Require Export BinInt Zcompare Zorder ZBinary. diff --git a/theories/ZArith/Zmin.v b/theories/ZArith/Zmin.v index e1599d943..317f912eb 100644 --- a/theories/ZArith/Zmin.v +++ b/theories/ZArith/Zmin.v @@ -5,8 +5,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** THIS FILE IS DEPRECATED. Use [ZBinary.Z] instead. *) Require Import BinInt Zcompare Zorder ZBinary. diff --git a/theories/ZArith/Zmisc.v b/theories/ZArith/Zmisc.v index 178ae5f15..820ed4a69 100644 --- a/theories/ZArith/Zmisc.v +++ b/theories/ZArith/Zmisc.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Wf_nat. Require Import BinInt. Require Import Zcompare. diff --git a/theories/ZArith/Znat.v b/theories/ZArith/Znat.v index dfd9b5450..1ca476d35 100644 --- a/theories/ZArith/Znat.v +++ b/theories/ZArith/Znat.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) Require Export Arith_base. diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v index 2a2751c9d..82ea3e94a 100644 --- a/theories/ZArith/Znumtheory.v +++ b/theories/ZArith/Znumtheory.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith_base. Require Import ZArithRing. Require Import Zcomplements. diff --git a/theories/ZArith/Zorder.v b/theories/ZArith/Zorder.v index 511c364bc..d2c8d9c04 100644 --- a/theories/ZArith/Zorder.v +++ b/theories/ZArith/Zorder.v @@ -6,8 +6,6 @@ (* // * This file is distributed under the terms of the *) (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) Require Import BinPos. diff --git a/theories/ZArith/Zpow_facts.v b/theories/ZArith/Zpow_facts.v index 1d9b3dfc9..43190ed05 100644 --- a/theories/ZArith/Zpow_facts.v +++ b/theories/ZArith/Zpow_facts.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import ZArith_base. Require Import ZArithRing. Require Import Zcomplements. diff --git a/theories/ZArith/Zpower.v b/theories/ZArith/Zpower.v index 508e6601c..ad02acb23 100644 --- a/theories/ZArith/Zpower.v +++ b/theories/ZArith/Zpower.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - Require Import Wf_nat. Require Import ZArith_base. Require Export Zpow_def. diff --git a/theories/ZArith/Zsqrt.v b/theories/ZArith/Zsqrt.v index b845cf47a..79714114b 100644 --- a/theories/ZArith/Zsqrt.v +++ b/theories/ZArith/Zsqrt.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import ZArithRing. Require Import Omega. Require Export ZArith_base. diff --git a/theories/ZArith/Zwf.v b/theories/ZArith/Zwf.v index 32d6de19a..88a5a9a56 100644 --- a/theories/ZArith/Zwf.v +++ b/theories/ZArith/Zwf.v @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - Require Import ZArith_base. Require Export Wf_nat. Require Import Omega. diff --git a/theories/ZArith/auxiliary.v b/theories/ZArith/auxiliary.v index 7af99ece9..81584e1e3 100644 --- a/theories/ZArith/auxiliary.v +++ b/theories/ZArith/auxiliary.v @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) Require Export Arith_base. diff --git a/tools/coq_makefile.ml4 b/tools/coq_makefile.ml4 index 617ca1d97..a7c89e7af 100644 --- a/tools/coq_makefile.ml4 +++ b/tools/coq_makefile.ml4 @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* créer un Makefile pour un développement Coq automatiquement *) type target = diff --git a/tools/coq_tex.ml4 b/tools/coq_tex.ml4 index c46a187c5..ec5cc42df 100644 --- a/tools/coq_tex.ml4 +++ b/tools/coq_tex.ml4 @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* coq-tex * JCF, 16/1/98 * adapted from caml-tex (perl script written by Xavier Leroy) diff --git a/tools/coqdep.ml b/tools/coqdep.ml index fe930a1de..ea7982d8a 100644 --- a/tools/coqdep.ml +++ b/tools/coqdep.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Printf open Coqdep_lexer open Coqdep_common diff --git a/tools/coqdep_boot.ml b/tools/coqdep_boot.ml index 2798e4af6..a97ba22b0 100644 --- a/tools/coqdep_boot.ml +++ b/tools/coqdep_boot.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Coqdep_common (** [coqdep_boot] is a stripped-down version of [coqdep], whose diff --git a/tools/coqdep_common.ml b/tools/coqdep_common.ml index cb98bd413..cb6050fce 100644 --- a/tools/coqdep_common.ml +++ b/tools/coqdep_common.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id: coqdep_common.ml 11984 2009-03-16 13:41:49Z letouzey $ *) - open Printf open Coqdep_lexer open Unix diff --git a/tools/coqdep_lexer.mll b/tools/coqdep_lexer.mll index 74c556a7d..6c32d3de3 100755 --- a/tools/coqdep_lexer.mll +++ b/tools/coqdep_lexer.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - { open Filename diff --git a/tools/coqdoc/alpha.ml b/tools/coqdoc/alpha.ml index d25034f2a..18eae0211 100644 --- a/tools/coqdoc/alpha.ml +++ b/tools/coqdoc/alpha.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Cdglobals let norm_char_latin1 c = match Char.uppercase c with diff --git a/tools/coqdoc/alpha.mli b/tools/coqdoc/alpha.mli index 922a10d6c..285ed00a7 100644 --- a/tools/coqdoc/alpha.mli +++ b/tools/coqdoc/alpha.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Alphabetic order. *) val compare_char : char -> char -> int diff --git a/tools/coqdoc/cpretty.mli b/tools/coqdoc/cpretty.mli index 213c76aaf..09cc7b7c2 100644 --- a/tools/coqdoc/cpretty.mli +++ b/tools/coqdoc/cpretty.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Index val coq_file : string -> Cdglobals.coq_module -> unit diff --git a/tools/coqdoc/cpretty.mll b/tools/coqdoc/cpretty.mll index 56ee459ab..344d3af70 100644 --- a/tools/coqdoc/cpretty.mll +++ b/tools/coqdoc/cpretty.mll @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*s Utility functions for the scanners *) { diff --git a/tools/coqdoc/index.ml b/tools/coqdoc/index.ml index 889e5d6ff..9445c9606 100644 --- a/tools/coqdoc/index.ml +++ b/tools/coqdoc/index.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Filename open Lexing open Printf diff --git a/tools/coqdoc/index.mli b/tools/coqdoc/index.mli index 517ec97a7..bf9d906f3 100644 --- a/tools/coqdoc/index.mli +++ b/tools/coqdoc/index.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Cdglobals type loc = int diff --git a/tools/coqdoc/main.ml b/tools/coqdoc/main.ml index 67c63865a..f3ebe0dc3 100644 --- a/tools/coqdoc/main.ml +++ b/tools/coqdoc/main.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Modified by Lionel Elie Mamane on 9 & 10 Mar 2004: * - handling of absolute filenames (function coq_module) * - coq_module: chop ./// (arbitrary amount of slashes), not only "./" diff --git a/tools/coqdoc/output.ml b/tools/coqdoc/output.ml index 1892a0c9c..57e0afa43 100644 --- a/tools/coqdoc/output.ml +++ b/tools/coqdoc/output.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Cdglobals open Index diff --git a/tools/coqdoc/output.mli b/tools/coqdoc/output.mli index d836f6b39..67877af05 100644 --- a/tools/coqdoc/output.mli +++ b/tools/coqdoc/output.mli @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Cdglobals open Index diff --git a/tools/coqwc.mll b/tools/coqwc.mll index f3646a8a1..c539387bf 100644 --- a/tools/coqwc.mll +++ b/tools/coqwc.mll @@ -9,8 +9,6 @@ (* coqwc - counts the lines of spec, proof and comments in Coq sources * Copyright (C) 2003 Jean-Christophe Filliâtre *) -(*i $Id$ i*) - (*s {\bf coqwc.} Counts the lines of spec, proof and comments in a Coq source. It assumes the files to be lexically well-formed. *) diff --git a/tools/gallina.ml b/tools/gallina.ml index 8ba9ae104..6a0f23d38 100644 --- a/tools/gallina.ml +++ b/tools/gallina.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Gallina_lexer let vfiles = ref ([] : string list) diff --git a/tools/gallina_lexer.mll b/tools/gallina_lexer.mll index 6d35d8397..fe489459e 100644 --- a/tools/gallina_lexer.mll +++ b/tools/gallina_lexer.mll @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - { open Lexing diff --git a/toplevel/auto_ind_decl.ml b/toplevel/auto_ind_decl.ml index d8c7326a9..65eb45cb2 100644 --- a/toplevel/auto_ind_decl.ml +++ b/toplevel/auto_ind_decl.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* This file is about the automatic generation of schemes about decidable equality, created by Vincent Siles, Oct 2007 *) diff --git a/toplevel/autoinstance.ml b/toplevel/autoinstance.ml index b45e45c80..fe13f28ee 100644 --- a/toplevel/autoinstance.ml +++ b/toplevel/autoinstance.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id:$ *) - (*i*) open Pp open Printer diff --git a/toplevel/cerrors.ml b/toplevel/cerrors.ml index 130b0b591..4fe2dffa8 100644 --- a/toplevel/cerrors.ml +++ b/toplevel/cerrors.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Indtypes diff --git a/toplevel/cerrors.mli b/toplevel/cerrors.mli index 8f26f4495..4ef5401d8 100644 --- a/toplevel/cerrors.mli +++ b/toplevel/cerrors.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Util diff --git a/toplevel/class.ml b/toplevel/class.ml index 0166b5213..ec623f767 100644 --- a/toplevel/class.ml +++ b/toplevel/class.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Util open Pp open Names diff --git a/toplevel/class.mli b/toplevel/class.mli index 4ee894cc9..51fb8b26e 100644 --- a/toplevel/class.mli +++ b/toplevel/class.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Classops diff --git a/toplevel/classes.ml b/toplevel/classes.ml index b7860c8b0..40d44432e 100644 --- a/toplevel/classes.ml +++ b/toplevel/classes.ml @@ -7,8 +7,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (*i*) open Names open Decl_kinds diff --git a/toplevel/classes.mli b/toplevel/classes.mli index 279622843..cae779b08 100644 --- a/toplevel/classes.mli +++ b/toplevel/classes.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Decl_kinds open Term diff --git a/toplevel/command.ml b/toplevel/command.ml index 51c7e50a4..fcc6c8ace 100644 --- a/toplevel/command.ml +++ b/toplevel/command.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Flags diff --git a/toplevel/command.mli b/toplevel/command.mli index 904a1a034..446cdc1b3 100644 --- a/toplevel/command.mli +++ b/toplevel/command.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/toplevel/coqinit.ml b/toplevel/coqinit.ml index d9fcdb247..a6cd938ae 100644 --- a/toplevel/coqinit.ml +++ b/toplevel/coqinit.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open System open Toplevel diff --git a/toplevel/coqinit.mli b/toplevel/coqinit.mli index 925859458..f209fd738 100644 --- a/toplevel/coqinit.mli +++ b/toplevel/coqinit.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Initialization. *) val set_debug : unit -> unit diff --git a/toplevel/coqtop.ml b/toplevel/coqtop.ml index a88ee3ba6..885f9ce9a 100644 --- a/toplevel/coqtop.ml +++ b/toplevel/coqtop.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open System diff --git a/toplevel/coqtop.mli b/toplevel/coqtop.mli index 0c43cc757..e4f1537a2 100644 --- a/toplevel/coqtop.mli +++ b/toplevel/coqtop.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** The Coq main module. The following function [start] will parse the command line, print the banner, initialize the load path, load the input state, load the files given on the command line, load the ressource file, diff --git a/toplevel/discharge.ml b/toplevel/discharge.ml index 4c21e4915..700328c8c 100644 --- a/toplevel/discharge.ml +++ b/toplevel/discharge.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Names open Util open Sign diff --git a/toplevel/discharge.mli b/toplevel/discharge.mli index b3636d717..03f831c23 100644 --- a/toplevel/discharge.mli +++ b/toplevel/discharge.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Sign open Cooking open Declarations diff --git a/toplevel/himsg.ml b/toplevel/himsg.ml index 0fb9a33b2..6c8847ff9 100644 --- a/toplevel/himsg.ml +++ b/toplevel/himsg.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Flags diff --git a/toplevel/himsg.mli b/toplevel/himsg.mli index 23c10767d..464c8f89c 100644 --- a/toplevel/himsg.mli +++ b/toplevel/himsg.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names open Indtypes diff --git a/toplevel/ind_tables.ml b/toplevel/ind_tables.ml index 447aeca48..845a5697a 100644 --- a/toplevel/ind_tables.ml +++ b/toplevel/ind_tables.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* File created by Vincent Siles, Oct 2007, extended into a generic support for generation of inductive schemes by Hugo Herbelin, Nov 2009 *) diff --git a/toplevel/indschemes.ml b/toplevel/indschemes.ml index b8f2986f3..a5d15a28a 100644 --- a/toplevel/indschemes.ml +++ b/toplevel/indschemes.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Created by Hugo Herbelin from contents related to inductive schemes initially developed by Christine Paulin (induction schemes), Vincent Siles (decidable equality and boolean equality) and Matthieu Sozeau diff --git a/toplevel/indschemes.mli b/toplevel/indschemes.mli index aab60a590..291b66776 100644 --- a/toplevel/indschemes.mli +++ b/toplevel/indschemes.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Term diff --git a/toplevel/lemmas.ml b/toplevel/lemmas.ml index f80fbf201..fb789798f 100644 --- a/toplevel/lemmas.ml +++ b/toplevel/lemmas.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Created by Hugo Herbelin from contents related to lemma proofs in file command.ml, Aug 2009 *) diff --git a/toplevel/lemmas.mli b/toplevel/lemmas.mli index 44502b4e4..55d7dcf2e 100644 --- a/toplevel/lemmas.mli +++ b/toplevel/lemmas.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.fix_expr ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Decl_kinds diff --git a/toplevel/metasyntax.ml b/toplevel/metasyntax.ml index 06b751c5f..65aac9769 100644 --- a/toplevel/metasyntax.ml +++ b/toplevel/metasyntax.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Flags open Util diff --git a/toplevel/metasyntax.mli b/toplevel/metasyntax.mli index 63272b7d3..f558fc4d1 100644 --- a/toplevel/metasyntax.mli +++ b/toplevel/metasyntax.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Util open Names open Libnames diff --git a/toplevel/mltop.ml4 b/toplevel/mltop.ml4 index ee4370305..509ecd89d 100644 --- a/toplevel/mltop.ml4 +++ b/toplevel/mltop.ml4 @@ -11,8 +11,6 @@ * camlp4deps will not work for this file unless Makefile system enhanced. *) -(* $Id$ *) - open Util open Pp open Flags diff --git a/toplevel/mltop.mli b/toplevel/mltop.mli index a03ad6242..9da357581 100644 --- a/toplevel/mltop.mli +++ b/toplevel/mltop.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** If there is a toplevel under Coq, it is described by the following record. *) type toplevel = { diff --git a/toplevel/record.ml b/toplevel/record.ml index c1c1a9671..d95c3657e 100644 --- a/toplevel/record.ml +++ b/toplevel/record.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/toplevel/record.mli b/toplevel/record.mli index d432bff6d..2090cf1e5 100644 --- a/toplevel/record.mli +++ b/toplevel/record.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Sign diff --git a/toplevel/search.ml b/toplevel/search.ml index 075c80c9a..353caa206 100644 --- a/toplevel/search.ml +++ b/toplevel/search.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/toplevel/search.mli b/toplevel/search.mli index a9d62c6ef..28096eb5e 100644 --- a/toplevel/search.mli +++ b/toplevel/search.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Names open Term diff --git a/toplevel/toplevel.ml b/toplevel/toplevel.ml index ee821a48d..453552273 100644 --- a/toplevel/toplevel.ml +++ b/toplevel/toplevel.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Flags diff --git a/toplevel/toplevel.mli b/toplevel/toplevel.mli index f51c088f0..8980ef92b 100644 --- a/toplevel/toplevel.mli +++ b/toplevel/toplevel.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Pp open Pcoq diff --git a/toplevel/usage.ml b/toplevel/usage.ml index 257660481..d12cbb762 100644 --- a/toplevel/usage.ml +++ b/toplevel/usage.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - let version () = Printf.printf "The Coq Proof Assistant, version %s (%s)\n" Coq_config.version Coq_config.date; diff --git a/toplevel/usage.mli b/toplevel/usage.mli index 1dfd4897b..23e807c16 100644 --- a/toplevel/usage.mli +++ b/toplevel/usage.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** {6 Prints the version number on the standard output and exits (with 0). } *) val version : unit -> 'a diff --git a/toplevel/vernac.ml b/toplevel/vernac.ml index 0bdb68f49..8386dd2b3 100644 --- a/toplevel/vernac.ml +++ b/toplevel/vernac.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - (* Parsing of vernacular. *) open Pp diff --git a/toplevel/vernac.mli b/toplevel/vernac.mli index 8ae319791..01852f130 100644 --- a/toplevel/vernac.mli +++ b/toplevel/vernac.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Parsing of vernacular. *) (** Read a vernac command on the specified input (parse only). diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml index 36f1e96e9..1ec553a9a 100644 --- a/toplevel/vernacentries.ml +++ b/toplevel/vernacentries.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - (* Concrete syntax of the mathematical vernacular MV V2.6 *) open Pp diff --git a/toplevel/vernacentries.mli b/toplevel/vernacentries.mli index fa9f2b7c2..b70eb61fb 100644 --- a/toplevel/vernacentries.mli +++ b/toplevel/vernacentries.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Names open Term open Vernacinterp diff --git a/toplevel/vernacexpr.ml b/toplevel/vernacexpr.ml index e216f2520..cbd6fb8de 100644 --- a/toplevel/vernacexpr.ml +++ b/toplevel/vernacexpr.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id$ i*) - open Util open Names open Tacexpr diff --git a/toplevel/vernacinterp.ml b/toplevel/vernacinterp.ml index 0924e519b..040a153a6 100644 --- a/toplevel/vernacinterp.ml +++ b/toplevel/vernacinterp.ml @@ -6,8 +6,6 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* $Id$ *) - open Pp open Util open Names diff --git a/toplevel/vernacinterp.mli b/toplevel/vernacinterp.mli index 4c59eadba..0a58b17b5 100644 --- a/toplevel/vernacinterp.mli +++ b/toplevel/vernacinterp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - open Tacexpr (** Interpretation of extended vernac phrases. *) diff --git a/toplevel/whelp.ml4 b/toplevel/whelp.ml4 index 9d4b5ec0c..6919a9730 100644 --- a/toplevel/whelp.ml4 +++ b/toplevel/whelp.ml4 @@ -8,8 +8,6 @@ (*i camlp4deps: "parsing/grammar.cma" i*) -(* $Id$ *) - open Flags open Pp open Util diff --git a/toplevel/whelp.mli b/toplevel/whelp.mli index 4c14c836a..72245021d 100644 --- a/toplevel/whelp.mli +++ b/toplevel/whelp.mli @@ -6,8 +6,6 @@ * GNU Lesser General Public License Version 2.1 ***********************************************************************) -(*i $Id$ i*) - (** Coq interface to the Whelp query engine developed at the University of Bologna *) -- cgit v1.2.3