File tree Expand file tree Collapse file tree 3 files changed +27
-0
lines changed
Expand file tree Collapse file tree 3 files changed +27
-0
lines changed Original file line number Diff line number Diff line change 1+ #! /bin/env bash
2+ set -eu
3+
4+ W=/workspace/agda
5+ # Create container
6+ C=$( docker container create --rm -w $W ghcr.io/codewars/agda:latest agda --verbose=0 --include-path=. --library=standard-library --library=cubical ExampleTest.agda)
7+
8+ # Copy files from the current directory
9+ # example/Example.agda
10+ # example/ExampleTest.agda
11+ docker container cp example/. $C :$W
12+
13+ # Run tests
14+ docker container start --attach $C
Original file line number Diff line number Diff line change 1+ {-# OPTIONS --safe #-}
2+ module Example where
3+ open import Agda.Builtin.Equality
4+
5+ _⇆_ : {A : Set } {a b c : A} → a ≡ b → b ≡ c → a ≡ c
6+ refl ⇆ refl = refl
Original file line number Diff line number Diff line change 1+ {-# OPTIONS --safe #-}
2+ module ExampleTest where
3+ open import Agda.Builtin.Equality
4+ open import Example
5+
6+ check : {A : Set } {a b c : A} → a ≡ b → b ≡ c → a ≡ c
7+ check = _⇆_
You can’t perform that action at this time.
0 commit comments