Skip to content

Commit

Permalink
Added markdown titles to markdown files so they get built properly. N…
Browse files Browse the repository at this point in the history
…ot all of the titles are very interesting.
  • Loading branch information
ramsay-t committed May 9, 2024
1 parent f545b46 commit 8769a09
Show file tree
Hide file tree
Showing 51 changed files with 220 additions and 26 deletions.
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Algorithmic.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic
layout: page
---
```
module Algorithmic where
```
Expand Down Expand Up @@ -335,4 +339,4 @@ constr-cong' : ∀{Γ : Ctx Φ}{n}{i : Fin n}{A : Vec (List (Φ ⊢Nf⋆ *)) n}
→ (q : subst (IList (Γ ⊢_)) p' cs' ≡ subst (IList (Γ ⊢_)) p cs)
→ constr i A p' cs' ≡ constr i A p cs
constr-cong' refl refl refl = refl
```
```
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.BehaviouralEquivalence.CCvsCK
layout: page
---
# CK machine

```
Expand Down
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.BehaviouralEquivalence.CCvsCEK
layout: page
---
# CEK behavioural equivalence with CK machine

```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/CEK.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.CEK
layout: page
---
# CEK machine that discharges builtin args

```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/CK.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.CK
layout: page
---
# CK machine

```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Completeness.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Completeness
layout: page
---
```
module Algorithmic.Completeness where
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Erasure.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Erasure
layout: page
---
```
{-# OPTIONS --injective-type-constructors #-}
Expand Down
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Erasure.RenamingSubstitution
layout: page
---
```
module Algorithmic.Erasure.RenamingSubstitution where
```
Expand Down
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Algorithmic/Evaluation.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Evaluation
layout: page
---
```
module Algorithmic.Evaluation where
```
Expand Down Expand Up @@ -85,4 +89,4 @@ stepper {A} t n with eval (gas n) t
... | steps x (error _) = return (error A)
```


4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Examples.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Examples
layout: page
---
```
module Algorithmic.Examples where
```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Properties.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Properties
layout: page
---
```
module Algorithmic.Properties where
```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Reduction.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Reduction
layout: page
---
```
module Algorithmic.Reduction where
```
Expand Down
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Algorithmic/ReductionEC.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.ReductionEC
layout: page
---
```
module Algorithmic.ReductionEC where
```
Expand Down Expand Up @@ -371,4 +375,4 @@ ival : ∀ b → Value (builtin b / refl)
ival b = V-I b base
-- -}
```


Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.ReductionEC.Determinism
layout: page
---
```
module Algorithmic.ReductionEC.Determinism where
```
Expand Down Expand Up @@ -684,4 +688,4 @@ determinism {L = L} (ruleErr E' p) (ruleErr E'' q) | step ¬VL E err r' U with U
... | refl ,, refl ,, refl | refl ,, refl ,, refl = refl
-- -}
```


Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.ReductionEC.Progress
layout: page
---
```
module Algorithmic.ReductionEC.Progress where
```
Expand Down Expand Up @@ -139,4 +143,4 @@ progress (case M cases) with progress M
... | step (ruleErr E refl) = step (ruleErr (case cases E) refl)
... | done (V-constr e Tss refl refl vs refl) = step (ruleEC [] (β-case e Tss refl vs refl cases) refl refl)
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.RenamingSubstitution
layout: page
---
```
module Algorithmic.RenamingSubstitution where
```
Expand Down Expand Up @@ -591,4 +595,4 @@ exts⋆ˢ : ∀{Φ}{Γ Δ : Ctx Φ}
-}
```



7 changes: 5 additions & 2 deletions plutus-metatheory/src/Algorithmic/Signature.lagda.md
Original file line number Diff line number Diff line change
@@ -1,4 +1,7 @@

---
title: Algorithmic.Signature
layout: page
---
```
module Algorithmic.Signature where
```
Expand Down Expand Up @@ -94,4 +97,4 @@ uniqueSigTy (bresult _) (bresult _) = refl
uniqueSigTy (A B⇒ s) (.A B⇒ s') = cong (A B⇒_) (uniqueSigTy s s')
uniqueSigTy (sucΠ s) (sucΠ s') = cong sucΠ (uniqueSigTy s s')
```


4 changes: 4 additions & 0 deletions plutus-metatheory/src/Algorithmic/Soundness.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Algorithmic.Soundness
layout: page
---
```
module Algorithmic.Soundness where
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Builtin/Constant/AtomicType.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Builtin.Constant.AtomicType
layout: page
---

```
module Builtin.Constant.AtomicType where
Expand Down
1 change: 1 addition & 0 deletions plutus-metatheory/src/Check.lagda.md
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
---
title: Type Checker
layout: page
---
## Type checker
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Cost.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Cost
layout: page
---
# Costs


Expand Down
7 changes: 5 additions & 2 deletions plutus-metatheory/src/Cost/Base.lagda.md
Original file line number Diff line number Diff line change
@@ -1,4 +1,7 @@

---
title: Cost.Base
layout: page
---
```
module Cost.Base where
Expand Down Expand Up @@ -92,4 +95,4 @@ record MachineParameters (Cost : Set) : Set where
startupCost : Cost
startupCost = cekMachineCost BStartup
```
```
5 changes: 4 additions & 1 deletion plutus-metatheory/src/Cost/Model.lagda.md
Original file line number Diff line number Diff line change
@@ -1,4 +1,7 @@

---
title: Cost.Model
layout: page
---
# Builtin Cost Models

```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Cost/Raw.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Cost.Raw
layout: page
---
# Raw Cost structures to inferface with Haskell

```
Expand Down
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Cost/Size.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Cost.Size
layout: page
---
# Size of Constants

```
Expand Down Expand Up @@ -83,4 +87,4 @@ defaultConstantMeasure (tmCon (pair t u) (x , y)) =
defaultValueMeasure : Value → CostingNat
defaultValueMeasure (V-con ty x) = defaultConstantMeasure (tmCon ty x)
defaultValueMeasure _ = 0
```
```
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: ChurchNat
layout: page
---
```
module Declarative.Examples.StdLib.ChurchNat where
```
Expand Down
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Function
layout: page
---
```
module Declarative.Examples.StdLib.Function where
```
Expand Down
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Nat
layout: page
---
```
module Declarative.Examples.StdLib.Nat where
```
Expand Down
7 changes: 5 additions & 2 deletions plutus-metatheory/src/Evaluator/Base.lagda.md
Original file line number Diff line number Diff line change
@@ -1,4 +1,7 @@

---
title: Base
layout: page
---
```
module Evaluator.Base where
Expand Down Expand Up @@ -104,4 +107,4 @@ reportError (runtimeError runtimeTypeError) = "runtimeTypeError"
```
maxsteps : Nat
maxsteps = 10000000000
```
```
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Evaluator/Program.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Program Evaluators
layout: page
---
# Evaluators for Programs

```
Expand Down Expand Up @@ -227,4 +231,4 @@ typeCheckProgramN namedprog = do
-}
return (prettyPrintTy (unshifterTy Z (extricateScopeTy (extricateNf⋆ A))))
```


6 changes: 5 additions & 1 deletion plutus-metatheory/src/Evaluator/Term.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Term - Haskell Interface to the Metatheory
layout: page
---
# Haskell Interface to the metatheory

This module contains functions that are meant to be called from Haskell code.
Expand Down Expand Up @@ -336,4 +340,4 @@ alphaU plc1 plc2 | inj₂ plc1' | inj₂ plc2' | _ | _ = Bool.false
alphaU plc1 plc2 | _ | _ = Bool.false
{-# COMPILE GHC alphaU as alphaU #-}
```
```
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Main.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Main
layout: page
---
```
module Main where
Expand Down
6 changes: 5 additions & 1 deletion plutus-metatheory/src/Raw.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Raw
layout: page
---
```
module Raw where
```
Expand Down Expand Up @@ -180,4 +184,4 @@ rawListPrinter [] = ""
rawListPrinter (x ∷ []) = rawPrinter x
rawListPrinter (x ∷ y ∷ xs) = rawPrinter x ++ " , " ++ rawListPrinter (y ∷ xs)
```


4 changes: 4 additions & 0 deletions plutus-metatheory/src/RawU.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Raw - Interface to Haskell
layout: page
---

This module provides the interface between the Haskell code and the Agda code.
It replicates the Haskell representation of Raw. In particular, for term constants,
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Scoped.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Scoped
layout: page
---
```
module Scoped where
```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Scoped/Extrication.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Scoped.Extrication
layout: page
---
```
module Scoped.Extrication where
```
Expand Down
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Scoped.Extrication.RenamingSubstitution
layout: page
---
```
module Scoped.Extrication.RenamingSubstitution where
```
Expand Down
4 changes: 4 additions & 0 deletions plutus-metatheory/src/Scoped/RenamingSubstitution.lagda.md
Original file line number Diff line number Diff line change
@@ -1,3 +1,7 @@
---
title: Scoped.RenamingSubstitution
layout: page
---
```
module Scoped.RenamingSubstitution where
```
Expand Down

0 comments on commit 8769a09

Please sign in to comment.