Skip to content

Commit 25f0d62

Browse files
committed
Add copyright
1 parent 384811c commit 25f0d62

File tree

18 files changed

+108
-0
lines changed

18 files changed

+108
-0
lines changed

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Debruijn.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Intrinsically scoped de Bruijn indices
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Eval.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Big-step evaluator for System F<:
39
-/

Cslib/Computability/LambdaCalculus/WellScoped/FSub/RebindTheory/Core.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Rebinding morphisms
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/RebindTheory/TypeSystem.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
import Cslib.Computability.LambdaCalculus.WellScoped.FSub.RebindTheory.Core
28
import Cslib.Computability.LambdaCalculus.WellScoped.FSub.TypeSystem
39
import Cslib.Computability.LambdaCalculus.WellScoped.FSub.Substitution.Properties

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Reduce.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Operational semantics for System F<:
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/RetypeTheory/Core.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Retyping morphisms
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/RetypeTheory/TypeSystem.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
import Cslib.Computability.LambdaCalculus.WellScoped.FSub.RetypeTheory.Core
28

39
/-- Context retyping preserves subtyping judgments. -/

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Substitution.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Parallel substitution for System F<:
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Substitution/Core.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Parallel substitution for System F<:
39

Cslib/Computability/LambdaCalculus/WellScoped/FSub/Substitution/Properties.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,9 @@
1+
/-
2+
Copyright (c) 2025 Yichen Xu. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Yichen Xu.
5+
-/
6+
17
/-
28
# Properties of parallel substitution for System F<:
39

0 commit comments

Comments
 (0)