Skip to content

Commit

Permalink
LeYoneda: clean detritus; polish README
Browse files Browse the repository at this point in the history
  • Loading branch information
artagnon committed Oct 12, 2024
1 parent 5749678 commit b177e65
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 22 deletions.
10 changes: 4 additions & 6 deletions README.md
Original file line number Diff line number Diff line change
Expand Up @@ -13,13 +13,11 @@ Some features of this project:

Our axioms are:

```text
Section Variables:
side : HSet
```coq
Axioms:
functional_extensionality_dep
: forall (A : Type) (B : A -> Type) (f g : forall x : A, B x),
(forall x : A, f x = g x) -> f = g
functional_extensionality_dep
: forall (A : Type) (B : A -> Type) (f g : forall x : A, B x),
(forall x : A, f x = g x) -> f = g
```

## Current status
Expand Down
16 changes: 0 additions & 16 deletions theories/νType/LeYoneda.v
Original file line number Diff line number Diff line change
Expand Up @@ -353,20 +353,4 @@ Ltac solve_leY :=
| [ |- ?c ] => debug ltac:(idtac "Not a leY:" c); fail
end.

Example ex1 (n p q r : nat)
(Hpr : p.+2 <= r.+2)
(Hrq : r.+2 <= q.+2)
(Hq : q.+2 <= n) : forall C, (p.+1 <= q.+2 -> p.+1 <= q.+1 -> p.+2 <= r.+2 -> p.+2 <= n -> C) -> C.
intros C H. apply H.
solve_leY.
solve_leY.
solve_leY.
solve_leY.
Qed.

Hint Extern 0 (leY _ _) => solve_leY : typeclass_instances.

Example ex2 {n} p q r {Hpr : p.+2 <= r.+2} {Hrq : r.+2 <= q.+2} {Hq : q.+2 <= n}
{H: forall p q r, p.+1 <= r.+1 -> r <= q -> q <= n -> p <= n}: p <= n.
now apply (H p q r _ _ _).
Qed.

0 comments on commit b177e65

Please sign in to comment.