Skip to content

Commit

Permalink
chore: copyright header housekeeping and CI
Browse files Browse the repository at this point in the history
  • Loading branch information
david-christiansen committed Mar 21, 2024
1 parent 01cd34e commit 624d174
Show file tree
Hide file tree
Showing 32 changed files with 158 additions and 10 deletions.
20 changes: 20 additions & 0 deletions .github/workflows/copyright-header.yml
Original file line number Diff line number Diff line change
@@ -0,0 +1,20 @@
name: Check for copyright header

on: [pull_request]

jobs:
check-lean-files:
runs-on: ubuntu-latest
steps:
- uses: actions/checkout@v4

- name: Verify .lean files start with a copyright header.
run: |
FILES=$(find ./src -type f -name "*.lean" -exec perl -ne 'BEGIN { $/ = undef; } print "$ARGV\n" if !m{\A/-\nCopyright}; exit;' {} \;)
if [ -n "$FILES" ]; then
echo "Found .lean files which do not have a copyright header:"
echo "$FILES"
exit 1
else
echo "All copyright headers present."
fi
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import SubVerso.Highlighting
import SubVerso.Examples

Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Basic.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

import SubVerso.Highlighting
Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Generate.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Genre.Blog.Basic
import Verso.Genre.Blog.Template
import Verso.Genre.Blog.Theme
Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/LexedText.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean
import Verso.Parser

Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Site.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Doc
import Verso.Genre.Blog.Basic

Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Site/Syntax.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

import Verso.Genre.Blog.Site
Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Template.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

import SubVerso.Highlighting
Expand Down
6 changes: 6 additions & 0 deletions src/verso-blog/Verso/Genre/Blog/Theme.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Genre.Blog.Site
import Verso.Genre.Blog.Template

Expand Down
6 changes: 6 additions & 0 deletions src/verso-manual/Verso/Genre/Manual.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Doc
import Verso.Doc.Concrete
import Verso.Doc.TeX
Expand Down
6 changes: 6 additions & 0 deletions src/verso-manual/Verso/Genre/Manual/Html.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Output.Html

namespace Verso.Genre.Manual.Html
Expand Down
6 changes: 6 additions & 0 deletions src/verso-manual/Verso/Genre/Manual/Html/Style.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

namespace Verso.Genre.Manual.Html.Css

def pageStyle : String := r####"
Expand Down
6 changes: 6 additions & 0 deletions src/verso-manual/Verso/Genre/Manual/Slug.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean
import Verso.Method

Expand Down
6 changes: 6 additions & 0 deletions src/verso-manual/Verso/Genre/Manual/TeX.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

namespace Verso.Genre.Manual.TeX

def preamble (title : String) (authors : List String) (date : String) : String :=
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

-- This module serves as the root of the `Verso` library.
-- Import modules here that should be built as part of the library.
import Verso.Build
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso/Build.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

import Verso.Doc
Expand Down
3 changes: 2 additions & 1 deletion src/verso/Verso/Doc.lean
Original file line number Diff line number Diff line change
@@ -1,8 +1,9 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

namespace Verso
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso/Doc/ArgParse.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean
import Verso.Doc
import Verso.Hover
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Concrete.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Elab.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Elab/ExpanderAttribute.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Elab/InlineString.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Elab/Monad.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Html.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Doc/Lsp.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso/Doc/Suggestion.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

namespace Verso.Doc.Suggestion
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso/Doc/TeX.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Doc
import Verso.Method
import Verso.Output.TeX
Expand Down
6 changes: 6 additions & 0 deletions src/verso/Verso/Hover.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

namespace Verso.Hover
Expand Down
7 changes: 7 additions & 0 deletions src/verso/Verso/Output.lean
Original file line number Diff line number Diff line change
@@ -1 +1,8 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Verso.Output.Html
import Verso.Output.TeX
6 changes: 6 additions & 0 deletions src/verso/Verso/Output/TeX.lean
Original file line number Diff line number Diff line change
@@ -1,3 +1,9 @@
/-
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/

import Lean

open Lean
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Parser.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down
2 changes: 1 addition & 1 deletion src/verso/Verso/Syntax.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
/-
Copyright (c) 2023 Lean FRO LLC. All rights reserved.
Copyright (c) 2023-2024 Lean FRO LLC. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: David Thrane Christiansen
-/
Expand Down

0 comments on commit 624d174

Please sign in to comment.