Skip to content

Commit cb6e1ee

Browse files
committed
test file
1 parent 5948613 commit cb6e1ee

File tree

1 file changed

+21
-0
lines changed

1 file changed

+21
-0
lines changed
Lines changed: 21 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,21 @@
1+
open List
2+
3+
example : [3,1,4,2] ~ [2,4,1,3] := by grind
4+
5+
example (xs ys zs : List Nat) (h₁ : xs ⊆ ys) (h₂ : ys ~ zs) : xs ⊆ zs := by grind
6+
example (xs ys zs : List Nat) (h₁ : xs <+ ys) (h₂ : ys ~ zs) : xs ⊆ zs := by grind
7+
example (xs ys zs : List Nat) (h₁ : xs ~ ys) (h₂ : ys ~ zs) : xs ~ zs := by grind
8+
9+
example : List.range 10 ~ (List.range 5 ++ List.range' 5 5).reverse := by grind
10+
11+
variable [BEq α] [LawfulBEq α]
12+
13+
example (xs ys : List (List α)) (h : xs ~ ys) : xs.flatten ~ ys.flatten := by grind
14+
15+
example {l l' : List α} (hl : l ~ l') (_ : l'.Nodup) : l.Nodup := by grind
16+
17+
example {a b : α} {as bs : List α} :
18+
a :: as ++ b :: bs ~ b :: as ++ a :: bs := by grind
19+
20+
example (x y : α) (l : List α) :
21+
List.insert x (List.insert y l) ~ List.insert y (List.insert x l) := by grind

0 commit comments

Comments
 (0)